diff options
author | Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr> | 2014-11-21 16:47:03 +0100 |
---|---|---|
committer | Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr> | 2014-11-21 16:47:03 +0100 |
commit | 9f9ad7a56d719cec729038156c01c11595eb951a (patch) | |
tree | 089607d9a15ef4a70411e35e3668f47132bef372 /test-suite | |
parent | 9a56644b05248d2068f1c5f804e581bc8a7f7275 (diff) |
Adding test for bug #3424.
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/3424.v | 23 |
1 files changed, 23 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3424.v b/test-suite/bugs/closed/3424.v new file mode 100644 index 000000000..f9b2c3861 --- /dev/null +++ b/test-suite/bugs/closed/3424.v @@ -0,0 +1,23 @@ +Set Universe Polymorphism. +Inductive paths {A : Type} (a : A) : A -> Type := idpath : paths a a where "x = y" := (@paths _ x y) : type_scope. +Class Contr_internal (A : Type) := BuildContr { center : A ; contr : (forall y : A, center = y) }. +Inductive trunc_index : Type := minus_two | trunc_S (x : trunc_index). +Bind Scope trunc_scope with trunc_index. +Fixpoint IsTrunc_internal (n : trunc_index) (A : Type) : Type := + match n with + | minus_two => Contr_internal A + | trunc_S n' => forall (x y : A), IsTrunc_internal n' (x = y) + end. +Notation minus_one:=(trunc_S minus_two). +Notation "0" := (trunc_S minus_one) : trunc_scope. +Class IsTrunc (n : trunc_index) (A : Type) : Type := Trunc_is_trunc : IsTrunc_internal n A. +Notation IsHProp := (IsTrunc minus_one). +Notation IsHSet := (IsTrunc 0). +Goal forall (A : Type) (a b : A) (H' : IsHSet A), { x : Type & IsHProp x }. +Proof. +intros. +eexists. +(* exact (H' a b). *) +(* Undo. *) +apply (H' a b). +Qed. |