aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_089.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_089.v
parent3f64bd23a343bcd7be0ef07afa7d9e3249df24ec (diff)
Move opened bugs to bugs/opened
Diffstat (limited to 'test-suite/bugs/closed/HoTT_coq_089.v')
-rw-r--r--test-suite/bugs/closed/HoTT_coq_089.v42
1 files changed, 0 insertions, 42 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_089.v b/test-suite/bugs/closed/HoTT_coq_089.v
deleted file mode 100644
index 54ae4704a..000000000
--- a/test-suite/bugs/closed/HoTT_coq_089.v
+++ /dev/null
@@ -1,42 +0,0 @@
-Set Universe Polymorphism.
-Set Printing Universes.
-
-Inductive type_paths (A : Type) : Type -> Prop
- := idtypepath : type_paths A A.
-Monomorphic Definition comp_type_paths := Eval compute in type_paths.
-Check comp_type_paths.
-(* comp_type_paths
- : Type (* Top.12 *) -> Type (* Top.12 *) -> Prop *)
-(* This is terrible. *)
-
-Inductive type_paths' (A : Type) : Type -> Prop
- := idtypepath' : type_paths' A A
- | other_type_path : False -> forall B : Set, type_paths' A B.
-Monomorphic Definition comp_type_paths' := Eval compute in type_paths'.
-Check comp_type_paths'.
-(* comp_type_paths'
- : Type (* Top.24 *) -> Type (* Top.23 *) -> Prop *)
-(* Ok, then ... *)
-
-(** Fail if it's [U0 -> U0 -> _], but not on [U0 -> U1 -> _]. *)
-Goal Type.
-Proof.
- match type of comp_type_paths' with
- | ?U0 -> ?U1 -> ?R
- => exact (@comp_type_paths' nat U0)
- end.
-Defined.
-
-Goal Type.
-Proof.
- match type of comp_type_paths with
- | ?U0 -> ?U1 -> ?R
- => exact (@comp_type_paths nat U0)
- end.
- (* Toplevel input, characters 110-112:
-Error:
-The term "Type (* Top.51 *)" has type "Type (* Top.51+1 *)"
-while it is expected to have type "Type (* Top.51 *)"
-(Universe inconsistency: Cannot enforce Top.51 < Top.51 because Top.51
-= Top.51)). *)
-Defined.