aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-10-01 16:46:08 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2015-10-02 15:54:13 +0200
commit6b9ff2261c738ff8ce47b75e5ced2b85476b6210 (patch)
tree8a984c1551b4deb8316a3781fd9eb0a688fdc813 /test-suite/bugs
parentcbcf55ca44b5374f39979ced88061c82c03901b3 (diff)
Univs: fix test-suite file for #4287, now properly rejected.
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/4287.v52
1 files changed, 2 insertions, 50 deletions
diff --git a/test-suite/bugs/closed/4287.v b/test-suite/bugs/closed/4287.v
index 732f19f33..e139c5b6c 100644
--- a/test-suite/bugs/closed/4287.v
+++ b/test-suite/bugs/closed/4287.v
@@ -100,35 +100,15 @@ End Hurkens.
Polymorphic Record box (T : Type) := wrap {unwrap : T}.
-(* Here we instantiate to Prop *)
-(* Here we instantiate to Prop *)
+(* Here we instantiate to Set *)
-Fail Definition down (x : Type) : Set := box x.
-Definition down (x : Set) : Set := box x.
+Fail Definition down (x : Type) : Prop := box x.
Definition up (x : Prop) : Type := x.
Fail Definition back A : up (down A) -> A := unwrap A.
Fail Definition forth A : A -> up (down A) := wrap A.
-(* Lemma backforth (A:Type) (P:A->Type) (a:A) : *)
-(* P (back A (forth A a)) -> P a. *)
-(* Proof. *)
-(* intros; assumption. *)
-(* Qed. *)
-
-(* Lemma backforth_r (A:Type) (P:A->Type) (a:A) : *)
-(* P a -> P (back A (forth A a)). *)
-(* Proof. *)
-(* intros; assumption. *)
-(* Qed. *)
-
-(* Theorem bad : False. *)
-(* apply (paradox down up back forth backforth backforth_r). *)
-(* Qed. *)
-
-(* Print Assumptions bad. *)
-
Definition id {A : Type} (a : A) := a.
Definition setlt (A : Type@{i}) :=
let foo := Type@{i} : Type@{j} in True.
@@ -142,31 +122,3 @@ Check @setle@{Prop j}.
Fail Definition foo := @setle@{j Prop}.
Definition foo := @setle@{Prop j}.
-
-(* Definition up (x : Prop) : Type := x. *)
-
-(* Definition back A : up (down A) -> A := unwrap A. *)
-
-(* Definition forth A : A -> up (down A) := wrap A. *)
-
-(* Lemma backforth (A:Type) (P:A->Type) (a:A) : *)
-(* P (back A (forth A a)) -> P a. *)
-(* Proof. *)
-(* intros; assumption. *)
-(* Qed. *)
-
-(* Lemma backforth_r (A:Type) (P:A->Type) (a:A) : *)
-(* P a -> P (back A (forth A a)). *)
-(* Proof. *)
-(* intros; assumption. *)
-(* Qed. *)
-
-(* Theorem bad : False. *)
-(* apply (paradox down up back forth backforth backforth_r). *)
-(* Qed. *)
-
-(* Print Assumptions bad. *)
-
-(* Polymorphic Record box (T : Type) := wrap {unwrap : T}. *)
-
-(* Definition down (x : Type) : Prop := box x. *)