diff options
author | Maxime Dénès <mail@maximedenes.fr> | 2017-06-01 08:31:23 +0200 |
---|---|---|
committer | Maxime Dénès <mail@maximedenes.fr> | 2017-06-01 08:31:23 +0200 |
commit | 26f813b51387a7b01627e98e0f46dd078b43d184 (patch) | |
tree | 28203dc25a2e6be5e55ef973a977236f487b97b7 /test-suite | |
parent | e7e0946401aa931ddca90d616a7968d548ab060f (diff) | |
parent | 0bba5da999dc8eeef75c7040562f687ce589ed11 (diff) |
Merge PR#710: Add test-suite checks for coqchk with constraints
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/coqchk/univ.v | 13 |
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/coqchk/univ.v b/test-suite/coqchk/univ.v index 84a4009d7..19eea94b1 100644 --- a/test-suite/coqchk/univ.v +++ b/test-suite/coqchk/univ.v @@ -33,3 +33,16 @@ Inductive finite_of_order T (D : T -> Type) (n : natural) := (rank_injective : injective_in T natural D rank) (rank_onto : forall i, equivalent (less_than i n) (in_image T natural D rank i)). + +(* Constraints *) +Universes i j. +Inductive constraint1 : (Type -> Type) -> Type := mk_constraint1 : constraint1 (fun x : Type@{i} => (x : Type@{j})). +Constraint i < j. +Inductive constraint2 : Type@{j} := mkc2 (_ : Type@{i}). +Universes i' j'. +Constraint i' = j'. +Inductive constraint3 : (Type -> Type) -> Type := mk_constraint3 : constraint3 (fun x : Type@{i'} => (x : Type@{j'})). +Inductive constraint4 : (Type -> Type) -> Type + := mk_constraint4 : let U1 := Type in + let U2 := Type in + constraint4 (fun x : U1 => (x : U2)). |