aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/polymorphism.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-30 21:55:24 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-04 15:48:31 +0200
commit86c6649382bb9e42281ffe956c627c6d3987559b (patch)
tree7d42f94d33c2ac2e4241ce92014abc0785aed6ca /test-suite/success/polymorphism.v
parentdd96b1e5e8d0eb9f93cff423b6f9cf900aee49d7 (diff)
- Force every universe level to be >= Prop, so one cannot "go under" it anymore.
- Finish the change to level-to-level substitutions, in the checker.
Diffstat (limited to 'test-suite/success/polymorphism.v')
-rw-r--r--test-suite/success/polymorphism.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/success/polymorphism.v b/test-suite/success/polymorphism.v
index fd299b43a..9167c9fcb 100644
--- a/test-suite/success/polymorphism.v
+++ b/test-suite/success/polymorphism.v
@@ -250,7 +250,7 @@ Fail Check fun A : Type => foo A.
Check fun A : Prop => foo A.
Fail Definition bar := fun A : Set => foo A.
-Check (let A := Type in foo (id A)).
+Fail Check (let A := Type in foo (id A)).
Definition fooS (A : Set) := A.