aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_115.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-17 17:55:00 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-17 17:55:00 +0200
commitba4289e55b376074bd782f6dc376a76e7efaec11 (patch)
tree25deb7a225eaaece366ea29d982933816103297d /test-suite/bugs/closed/HoTT_coq_115.v
parent258cbd1d2619cc5916dd570b95050e37c06fba77 (diff)
Fix a destArity that does not exactly match isArity in presence of let-ins.
Diffstat (limited to 'test-suite/bugs/closed/HoTT_coq_115.v')
-rw-r--r--test-suite/bugs/closed/HoTT_coq_115.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_115.v b/test-suite/bugs/closed/HoTT_coq_115.v
new file mode 100644
index 000000000..c1e133eeb
--- /dev/null
+++ b/test-suite/bugs/closed/HoTT_coq_115.v
@@ -0,0 +1 @@
+Inductive T : let U := Type in U := t. (* Anomaly: not an arity. Please report. *)