aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3808.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-02-14 12:54:36 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-02-14 12:58:05 +0100
commitea083ac106f048e64c1b57ddd37ac717236b8ecd (patch)
tree497b4d44d8814614ed7f9e2c6ec8c328d62963c6 /test-suite/bugs/closed/3808.v
parent7dc6dfee7eb641282f4268aea24c688da07470ee (diff)
Univs: When computing the level of an inductive including indices, lets
do not contribute. Fixes bug #3808.
Diffstat (limited to 'test-suite/bugs/closed/3808.v')
-rw-r--r--test-suite/bugs/closed/3808.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3808.v b/test-suite/bugs/closed/3808.v
new file mode 100644
index 000000000..6e19ddf8d
--- /dev/null
+++ b/test-suite/bugs/closed/3808.v
@@ -0,0 +1,2 @@
+Inductive Foo : (let enforce := (fun x => x) : Type@{j} -> Type@{i} in Type@{i})
+ := foo : Foo. \ No newline at end of file