aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/coqchk/cumulativity.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/coqchk/cumulativity.v')
-rw-r--r--test-suite/coqchk/cumulativity.v11
1 files changed, 10 insertions, 1 deletions
diff --git a/test-suite/coqchk/cumulativity.v b/test-suite/coqchk/cumulativity.v
index 3a8f9fa22..ecf9035bf 100644
--- a/test-suite/coqchk/cumulativity.v
+++ b/test-suite/coqchk/cumulativity.v
@@ -49,4 +49,13 @@ Section TpLower.
Fail Definition LowerTp : Tp@{j} -> Tp@{i} := fun x => x.
-End TpLower. \ No newline at end of file
+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