aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4293.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-05 16:04:43 -0500
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-11 19:13:52 +0100
commit2f56f0fcf21902bb1317f1d6f7ba4b593d712646 (patch)
tree66ac9f8f8e35cf2146b8e5f8bb02ec72c6c5f575 /test-suite/bugs/closed/4293.v
parent701a69732ef2abfc7384296e090a3e9bd7604bbd (diff)
Fix bug #4293: ensure let-ins do not contain algebraic universes in
their type annotation.
Diffstat (limited to 'test-suite/bugs/closed/4293.v')
-rw-r--r--test-suite/bugs/closed/4293.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4293.v b/test-suite/bugs/closed/4293.v
new file mode 100644
index 000000000..3671c931b
--- /dev/null
+++ b/test-suite/bugs/closed/4293.v
@@ -0,0 +1,7 @@
+Module Type Foo.
+Definition T := let X := Type in Type.
+End Foo.
+
+Module M : Foo.
+Definition T := let X := Type in Type.
+End M. \ No newline at end of file