aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4390.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-10-27 13:55:45 -0400
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-10-27 14:03:42 -0400
commited7af646f2e486b7e96812ba2335e644756b70fd (patch)
tree4f800531ad9238598d7c6231b6b165c167bd6c1f /test-suite/bugs/closed/4390.v
parent7bf9bbe2968802b48230d35d34c585201ee9e9b4 (diff)
Fix bugs 4389, 4390 and 4391 due to wrong handling of universe names
structure.
Diffstat (limited to 'test-suite/bugs/closed/4390.v')
-rw-r--r--test-suite/bugs/closed/4390.v37
1 files changed, 37 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4390.v b/test-suite/bugs/closed/4390.v
new file mode 100644
index 000000000..a96a13700
--- /dev/null
+++ b/test-suite/bugs/closed/4390.v
@@ -0,0 +1,37 @@
+Module A.
+Set Printing All.
+Set Printing Universes.
+
+Module M.
+Section foo.
+Universe i.
+End foo.
+End M.
+
+Check Type@{i}.
+(* Succeeds *)
+
+Fail Check Type@{j}.
+(* Error: Undeclared universe: j *)
+
+Definition foo@{j} : Type@{i} := Type@{j}.
+(* ok *)
+End A.
+
+Set Universe Polymorphism.
+Fail Universes j.
+Monomorphic Universe j.
+Section foo.
+ Universes i.
+ Constraint i < j.
+ Definition foo : Type@{j} := Type@{i}.
+ Definition foo' : Type@{j} := Type@{i}.
+End foo.
+
+Check eq_refl : foo@{i} = foo'@{i}.
+
+Definition bar := foo.
+Monomorphic Definition bar'@{k} := foo@{k}.
+
+Fail Constraint j = j.
+Monomorphic Constraint i = i.