aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-09 13:10:18 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-09 13:10:18 +0200
commitc3ce76de37a988c120654760629b4609272f8885 (patch)
tree8ad851468b3d0b9fb3bfd775f4c760af97c560f8 /test-suite/bugs
parent79220cec31a9c2c5cafc678b36f7af374417ecd5 (diff)
Refresh universes for Ltac's type_of, as the term can be used anywhere,
fixing two opened bugs from HoTT/coq.
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/HoTT_coq_074.v10
-rw-r--r--test-suite/bugs/closed/HoTT_coq_114.v1
-rw-r--r--test-suite/bugs/opened/HoTT_coq_074.v12
-rw-r--r--test-suite/bugs/opened/HoTT_coq_114.v2
4 files changed, 11 insertions, 14 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_074.v b/test-suite/bugs/closed/HoTT_coq_074.v
new file mode 100644
index 000000000..370c7d404
--- /dev/null
+++ b/test-suite/bugs/closed/HoTT_coq_074.v
@@ -0,0 +1,10 @@
+Monomorphic Definition U1 := Type.
+Monomorphic Definition U2 := Type.
+
+Set Printing Universes.
+Definition foo : True.
+let t1 := type of U1 in
+let t2 := type of U2 in
+idtac t1 t2;
+pose (t1 : t2). exact I.
+Defined.
diff --git a/test-suite/bugs/closed/HoTT_coq_114.v b/test-suite/bugs/closed/HoTT_coq_114.v
new file mode 100644
index 000000000..341128338
--- /dev/null
+++ b/test-suite/bugs/closed/HoTT_coq_114.v
@@ -0,0 +1 @@
+Inductive test : $(let U := type of Type in exact U)$ := t.
diff --git a/test-suite/bugs/opened/HoTT_coq_074.v b/test-suite/bugs/opened/HoTT_coq_074.v
deleted file mode 100644
index 7c88447b2..000000000
--- a/test-suite/bugs/opened/HoTT_coq_074.v
+++ /dev/null
@@ -1,12 +0,0 @@
-Monomorphic Definition U1 := Type.
-Monomorphic Definition U2 := Type.
-
-Set Printing Universes.
-Definition foo : True.
-Fail let t1 := type of U1 in
-let t2 := type of U2 in
-pose (t1 : t2). (* Error:
-The term "Type (* Top.1+1 *)" has type "Type (* Top.1+2 *)"
-while it is expected to have type "Type (* Top.2+1 *)". *)
-exact I.
-Defined.
diff --git a/test-suite/bugs/opened/HoTT_coq_114.v b/test-suite/bugs/opened/HoTT_coq_114.v
deleted file mode 100644
index e293e6dbb..000000000
--- a/test-suite/bugs/opened/HoTT_coq_114.v
+++ /dev/null
@@ -1,2 +0,0 @@
-Fail Inductive test : $(let U := type of Type in exact U)$ := t.
-(* Anomaly: Unable to handle arbitrary u+k <= v constraints. Please report. *)