diff src/GeneralRec.v @ 572:a913f19955e2

Update for Coq 8.11
author Adam Chlipala <adam@chlipala.net>
date Sun, 02 Feb 2020 10:46:14 -0500
parents 81d63d9c1cc5
children 1dc1d41620b6
line wrap: on
line diff
--- a/src/GeneralRec.v	Sun Apr 21 16:09:55 2019 -0400
+++ b/src/GeneralRec.v	Sun Feb 02 10:46:14 2020 -0500
@@ -781,6 +781,8 @@
 
 I know no easy fix for this problem of [thunk], but we can define an alternate co-inductive monad that avoids the problem, based on a proposal by Megacz%~\cite{Megacz}%.  We ran into trouble because [TBind] was not a constructor of [thunk], so let us define a new type family where "bind" is a constructor. *)
 
+Set Universe Polymorphism.
+
 CoInductive comp (A : Type) : Type :=
 | Ret : A -> comp A
 | Bnd : forall B, comp B -> (B -> comp A) -> comp A.