aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/polymorphism.v
diff options
context:
space:
mode:
authorGravatar Gaƫtan Gilbert <gaetan.gilbert@ens-lyon.fr>2017-06-12 17:47:51 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2017-09-19 10:28:03 +0200
commitd9e54d65cc808eab2908beb7a7a2c96005118ace (patch)
treeb214d227a3c5186dd512fb0f53064b4220ff2648 /test-suite/success/polymorphism.v
parentf72a67569ec8cb9160d161699302b67919da5686 (diff)
Allow declaring universe binders with no constraints with @{|}
Diffstat (limited to 'test-suite/success/polymorphism.v')
-rw-r--r--test-suite/success/polymorphism.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/test-suite/success/polymorphism.v b/test-suite/success/polymorphism.v
index 0bd8bfe60..488443de1 100644
--- a/test-suite/success/polymorphism.v
+++ b/test-suite/success/polymorphism.v
@@ -159,6 +159,8 @@ End structures.
Module binders.
+ Definition mynat@{|} := nat.
+
Definition foo@{i j | i < j, i < j} (A : Type@{i}) : Type@{j}.
exact A.
Defined.