aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2016-01-23 17:28:34 -0500
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2016-01-23 17:32:03 -0500
commitb582db2ecbb3f7f1315fedc50b0009f62f5c59ad (patch)
tree7124248152310d58c438d4ea0de69b3761f9e082 /theories/Logic
parent6a046f8d3e33701d70e2a391741e65564cc0554d (diff)
Fix bug #4503: mixing universe polymorphic and monomorphic
variables and definitions in sections is unsupported.
Diffstat (limited to 'theories/Logic')
-rw-r--r--theories/Logic/Hurkens.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/Logic/Hurkens.v b/theories/Logic/Hurkens.v
index 8ded74763..841f843c0 100644
--- a/theories/Logic/Hurkens.v
+++ b/theories/Logic/Hurkens.v
@@ -631,6 +631,8 @@ End NoRetractFromTypeToProp.
Module TypeNeqSmallType.
+Unset Universe Polymorphism.
+
Section Paradox.
(** ** Universe [U] is equal to one of its elements. *)
@@ -655,7 +657,6 @@ Proof.
reflexivity.
Qed.
-
Theorem paradox : False.
Proof.
Generic.paradox p.