aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Amin Timany <amintimany@gmail.com>2017-05-27 09:48:53 +0200
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-06-16 04:51:19 +0200
commit3380f47d2bb38d549fcdac8fb073f9aa1f259a23 (patch)
tree73a02774d323e09d4cc59173833a9a8e2db2c2b1
parent249a1910a2474216b7f98491afafc6019a04c894 (diff)
Move (part of) tests from checker to success
Due to some unknown problem coqchk fails on some inductive types when it is compiled with ocaml4.02.3+32bit and camlp5-4.16 which is the case for Travis tests.
-rw-r--r--test-suite/coqchk/cumulativity.v43
-rw-r--r--test-suite/success/cumulativity.v61
2 files changed, 86 insertions, 18 deletions
diff --git a/test-suite/coqchk/cumulativity.v b/test-suite/coqchk/cumulativity.v
index ecf9035bf..84121ea92 100644
--- a/test-suite/coqchk/cumulativity.v
+++ b/test-suite/coqchk/cumulativity.v
@@ -28,34 +28,41 @@ End ListLower.
Lemma LowerL_Lem@{i j} (A : Type@{j}) (l : List@{i} A) : l = LowerL l.
Proof. reflexivity. Qed.
-Inductive Tp := tp : Type -> Tp.
+(* I disable these tests because cqochk can't process them when compiled with
+ ocaml-4.02.3+32bit and camlp5-4.16 which is the case for Travis!
-Section TpLift.
- Universe i j.
+ I have added this file (including the commented parts below) in
+ test-suite/success/cumulativity.v which doesn't run coqchk on them.
+*)
- Constraint i < j.
+(* Inductive Tp := tp : Type -> Tp. *)
- Definition LiftTp : Tp@{i} -> Tp@{j} := fun x => x.
+(* Section TpLift. *)
+(* Universe i j. *)
-End TpLift.
+(* Constraint i < j. *)
-Lemma LiftC_Lem (t : Tp) : LiftTp t = t.
-Proof. reflexivity. Qed.
+(* Definition LiftTp : Tp@{i} -> Tp@{j} := fun x => x. *)
-Section TpLower.
- Universe i j.
+(* End TpLift. *)
- Constraint i < j.
+(* Lemma LiftC_Lem (t : Tp) : LiftTp t = t. *)
+(* Proof. reflexivity. Qed. *)
- Fail Definition LowerTp : Tp@{j} -> Tp@{i} := fun x => x.
+(* Section TpLower. *)
+(* Universe i j. *)
-End TpLower.
+(* Constraint i < j. *)
+(* Fail Definition LowerTp : Tp@{j} -> Tp@{i} := fun x => x. *)
-Section subtyping_test.
- Universe i j.
- Constraint i < j.
+(* End TpLower. *)
+
+
+(* Section subtyping_test. *)
+(* Universe i j. *)
+(* Constraint i < j. *)
- Inductive TP2 := tp2 : Type@{i} -> Type@{j} -> TP2.
+(* Inductive TP2 := tp2 : Type@{i} -> Type@{j} -> TP2. *)
-End subtyping_test. \ No newline at end of file
+(* End subtyping_test. *) \ No newline at end of file
diff --git a/test-suite/success/cumulativity.v b/test-suite/success/cumulativity.v
new file mode 100644
index 000000000..ecf9035bf
--- /dev/null
+++ b/test-suite/success/cumulativity.v
@@ -0,0 +1,61 @@
+Set Universe Polymorphism.
+Set Inductive Cumulativity.
+Set Printing Universes.
+
+Inductive List (A: Type) := nil | cons : A -> List A -> List A.
+
+Section ListLift.
+ Universe i j.
+
+ Constraint i < j.
+
+ Definition LiftL {A} : List@{i} A -> List@{j} A := fun x => x.
+
+End ListLift.
+
+Lemma LiftL_Lem A (l : List A) : l = LiftL l.
+Proof. reflexivity. Qed.
+
+Section ListLower.
+ Universe i j.
+
+ Constraint i < j.
+
+ Definition LowerL {A : Type@{i}} : List@{j} A -> List@{i} A := fun x => x.
+
+End ListLower.
+
+Lemma LowerL_Lem@{i j} (A : Type@{j}) (l : List@{i} A) : l = LowerL l.
+Proof. reflexivity. Qed.
+
+Inductive Tp := tp : Type -> Tp.
+
+Section TpLift.
+ Universe i j.
+
+ Constraint i < j.
+
+ Definition LiftTp : Tp@{i} -> Tp@{j} := fun x => x.
+
+End TpLift.
+
+Lemma LiftC_Lem (t : Tp) : LiftTp t = t.
+Proof. reflexivity. Qed.
+
+Section TpLower.
+ Universe i j.
+
+ Constraint i < j.
+
+ Fail Definition LowerTp : Tp@{j} -> Tp@{i} := fun x => x.
+
+End TpLower.
+
+
+Section subtyping_test.
+ Universe i j.
+ Constraint i < j.
+
+ Inductive TP2 := tp2 : Type@{i} -> Type@{j} -> TP2.
+
+End subtyping_test. \ No newline at end of file