diff options
| author | Emilio Jesus Gallego Arias | 2018-05-15 04:25:05 +0200 |
|---|---|---|
| committer | Emilio Jesus Gallego Arias | 2018-09-26 16:44:04 +0200 |
| commit | ef3fa51c12c450781facb61f54f465a77a359f83 (patch) | |
| tree | 583760a05d9530060f6ba9054c408d88fca6dc4a /test-suite | |
| parent | f49928874b51458fb67e89618bb350ae2f3529e4 (diff) | |
[ocaml] Update required OCaml version to 4.05.0
Closes #7380. Ubuntu 18.04 and Debian Buster will ship this OCaml
version so it makes sense we bump our dependency to 4.05.0 as we can
use some newer compiler features.
Diffstat (limited to 'test-suite')
| -rw-r--r-- | test-suite/coqchk/cumulativity.v | 42 |
1 files changed, 18 insertions, 24 deletions
diff --git a/test-suite/coqchk/cumulativity.v b/test-suite/coqchk/cumulativity.v index 034684054d..c3f6bebcbe 100644 --- a/test-suite/coqchk/cumulativity.v +++ b/test-suite/coqchk/cumulativity.v @@ -27,41 +27,35 @@ End ListLower. Lemma LowerL_Lem@{i j|j<i+} (A : Type@{j}) (l : List@{i} A) : l = LowerL@{j i} l. Proof. reflexivity. Qed. -(* -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! - I have added this file (including the commented parts below) in - test-suite/success/cumulativity.v which doesn't run coqchk on them. -*) -(* Inductive Tp := tp : Type -> Tp. *) +Inductive Tp := tp : Type -> Tp. -(* Section TpLift. *) -(* Universe i j. *) +Section TpLift. -(* Constraint i < j. *) + Universe i j. -(* Definition LiftTp : Tp@{i} -> Tp@{j} := fun x => x. *) + Constraint i < j. -(* End TpLift. *) + Definition LiftTp : Tp@{i} -> Tp@{j} := fun x => x. -(* Lemma LiftC_Lem (t : Tp) : LiftTp t = t. *) -(* Proof. reflexivity. Qed. *) +End TpLift. -(* Section TpLower. *) -(* Universe i j. *) +Lemma LiftC_Lem (t : Tp) : LiftTp t = t. +Proof. reflexivity. Qed. -(* Constraint i < j. *) +Section TpLower. + Universe i j. -(* Fail Definition LowerTp : Tp@{j} -> Tp@{i} := fun x => x. *) + Constraint i < j. -(* End TpLower. *) + Fail Definition LowerTp : Tp@{j} -> Tp@{i} := fun x => x. +End TpLower. -(* Section subtyping_test. *) -(* Universe i j. *) -(* Constraint i < j. *) +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. *) +End subtyping_test. |
