aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar Cyprien Mangin <cyprien.mangin@m4x.org>2018-06-14 16:29:19 +0200
committerGravatar Cyprien Mangin <cyprien.mangin@m4x.org>2018-06-14 16:29:19 +0200
commit2a239725f493e643d0f26455293e6ca295f4dc92 (patch)
tree046ed781a6e67f623da3d0eb88c03ffaee8843cb /test-suite/bugs
parent1098604f599aa9aae9f07cf4960f41ef34f865e5 (diff)
Workaround to handle non-value arguments in tactics.
Although the fix is not a proper one, it seems to solve every instance of #2800 that could be tested.
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/2800.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/2800.v b/test-suite/bugs/closed/2800.v
index 2ee438934..54c75e344 100644
--- a/test-suite/bugs/closed/2800.v
+++ b/test-suite/bugs/closed/2800.v
@@ -4,3 +4,16 @@ intuition
match goal with
| |- _ => idtac " foo"
end.
+
+ lazymatch goal with _ => idtac end.
+ match goal with _ => idtac end.
+ unshelve lazymatch goal with _ => idtac end.
+ unshelve match goal with _ => idtac end.
+ unshelve (let x := I in idtac).
+Abort.
+
+Require Import ssreflect.
+
+Goal True.
+match goal with _ => idtac end => //.
+Qed.