aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/5331.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-01-31 06:36:25 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-01-31 09:41:13 +0100
commitf5923c2174fbb419397f127af31ab1cd0b223e0a (patch)
tree3babfe486803cf4c0b27ed70f9b7f600ebb01f49 /test-suite/bugs/closed/5331.v
parenta0fb4f60bb328935da053250e7964150fdf57a86 (diff)
Fixing #5311 (anomaly on unexpected intro pattern).
This was introduced in 8.5 while reorganizing the structure of intro-patterns.
Diffstat (limited to 'test-suite/bugs/closed/5331.v')
-rw-r--r--test-suite/bugs/closed/5331.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5331.v b/test-suite/bugs/closed/5331.v
new file mode 100644
index 000000000..0d72fcb5d
--- /dev/null
+++ b/test-suite/bugs/closed/5331.v
@@ -0,0 +1,11 @@
+(* Checking no anomaly on some unexpected intropattern *)
+
+Ltac ih H := induction H as H.
+Ltac ih' H H' := induction H as H'.
+
+Goal True -> True.
+Fail intro H; ih H.
+intro H; ih' H ipattern:[].
+exact I.
+Qed.
+