aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_113.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2014-05-12 11:04:50 -0400
committerGravatar Jason Gross <jgross@mit.edu>2014-05-12 11:04:50 -0400
commit9c7e0a2e6a8e46dc439603cde501037a3e18050a (patch)
tree30466045fb87ba5e8d29adb1e658f1020bb70de3 /test-suite/bugs/closed/HoTT_coq_113.v
parent4a0e4ee76663a12e3cb3d22ce77b0d37a5830af5 (diff)
Update various polyproj bugs w.r.t. latest trunk
Diffstat (limited to 'test-suite/bugs/closed/HoTT_coq_113.v')
-rw-r--r--test-suite/bugs/closed/HoTT_coq_113.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_113.v b/test-suite/bugs/closed/HoTT_coq_113.v
new file mode 100644
index 000000000..3ef531bc9
--- /dev/null
+++ b/test-suite/bugs/closed/HoTT_coq_113.v
@@ -0,0 +1,19 @@
+(* File reduced by coq-bug-finder from original input, then from 3329 lines to 153 lines, then from 118 lines to 49 lines, then from 55 lines to 38 lines, then from 46 lines to 16 lines *)
+
+Generalizable All Variables.
+Set Universe Polymorphism.
+Class Foo (A : Type) := {}.
+Definition Baz := Foo.
+Definition Bar {A B} `{Foo A, Foo B} : True.
+Proof.
+ Set Printing Universes.
+ (* [change] should give fresh universes for each [Foo] *)
+ change Foo with Baz in *.
+ admit.
+Defined.
+Definition foo := @Bar nat.
+Check @foo Set.
+(* Toplevel input, characters 26-29:
+Error:
+The term "Set" has type "Type (* Set+1 *)" while it is expected to have type
+ "Set" (Universe inconsistency: Cannot enforce Set < Set because Set = Set)). *)