aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_113.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2014-05-09 10:13:32 -0400
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-10 15:39:39 +0200
commitc7284415e4bdd3315c84c7d15d140d3fee000bc5 (patch)
treecc8ded3feba7e1da0dd4f7d17b7e5f974de752c3 /test-suite/bugs/closed/HoTT_coq_113.v
parent3f64bd23a343bcd7be0ef07afa7d9e3249df24ec (diff)
Move opened bugs to bugs/opened
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, 0 insertions, 19 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_113.v b/test-suite/bugs/closed/HoTT_coq_113.v
deleted file mode 100644
index 3ef531bc9..000000000
--- a/test-suite/bugs/closed/HoTT_coq_113.v
+++ /dev/null
@@ -1,19 +0,0 @@
-(* 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)). *)