aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/polymorphism.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-04-07 17:29:26 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-06 09:58:59 +0200
commit2d6de8b102ea3cd05c5d193190faf787ccb84baa (patch)
tree876350b54e58c77b0bb265afa65a04acd0536872 /test-suite/success/polymorphism.v
parentd081f9390206c510d9837e2ecd3fa0a0d4ef0b8c (diff)
Fix restrict_universe_context removing some universes that do appear in the term.
Diffstat (limited to 'test-suite/success/polymorphism.v')
-rw-r--r--test-suite/success/polymorphism.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/success/polymorphism.v b/test-suite/success/polymorphism.v
index 7c1166c4c..1ef2713e4 100644
--- a/test-suite/success/polymorphism.v
+++ b/test-suite/success/polymorphism.v
@@ -243,7 +243,7 @@ Polymorphic Definition fun_ext (A B : Type) :=
Polymorphic Class Funext A B := extensional : fun_ext A B.
-Section foo.
+Section foo2.
Context `{forall A B, Funext A B}.
Print Universes.
-End foo.
+End foo2.