aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/5215_2.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2017-11-20 18:43:31 +0100
committerGravatar Matthieu Sozeau <mattam@mattam.org>2017-11-22 11:14:46 +0100
commit2db70092d63065be8a5902764e0d1d5f1ea01e6c (patch)
tree478c124734b6444141378a1df22488f77b2102c7 /test-suite/bugs/closed/5215_2.v
parent2a857da2a88855a6c9f0fa7e48a8700c1613e0c7 (diff)
Fix universe polymorphic Program obligations.
The universes of the obligations should all be non-algebraic as they might appear in instances of other obligations and instances only take non-algebraic universes as arguments.
Diffstat (limited to 'test-suite/bugs/closed/5215_2.v')
-rw-r--r--test-suite/bugs/closed/5215_2.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5215_2.v b/test-suite/bugs/closed/5215_2.v
new file mode 100644
index 000000000..399947f00
--- /dev/null
+++ b/test-suite/bugs/closed/5215_2.v
@@ -0,0 +1,8 @@
+Require Import Coq.Program.Tactics.
+Set Universe Polymorphism.
+Set Printing Universes.
+Definition typ := Type.
+
+Program Definition foo : typ := _ -> _.
+Next Obligation. Admitted.
+Next Obligation. exact typ. Show Proof. Show Universes. Defined.