aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorTej Chajed2020-02-23 08:02:11 -0500
committerGitHub2020-02-23 08:02:11 -0500
commit92d2004cc678091370a91037943ca7953bbb5c5d (patch)
tree60e00942e4c5be551adfc867688fc6b00d91809a
parent8e3ff397ed403f3da90300ec3196810167ce61a0 (diff)
parent5360fb1202375d90adde5c8ba6700098e57bed53 (diff)
Merge pull request #11629 from ppedrot/fix-11552
Fix #11552: Ltac2 breaks query commands during proofs.
-rw-r--r--test-suite/bugs/closed/bug_11552.v9
-rw-r--r--user-contrib/Ltac2/g_ltac2.mlg6
2 files changed, 15 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/bug_11552.v b/test-suite/bugs/closed/bug_11552.v
new file mode 100644
index 0000000000..189b1d9d8a
--- /dev/null
+++ b/test-suite/bugs/closed/bug_11552.v
@@ -0,0 +1,9 @@
+From Ltac2 Require Import Ltac2.
+
+Goal True.
+Proof.
+ Search unit.
+ (* Unbound constructor Search *)
+ Check tt.
+ (* Unbound constructor Check *)
+Abort.
diff --git a/user-contrib/Ltac2/g_ltac2.mlg b/user-contrib/Ltac2/g_ltac2.mlg
index c1bd585f3f..d05640f22d 100644
--- a/user-contrib/Ltac2/g_ltac2.mlg
+++ b/user-contrib/Ltac2/g_ltac2.mlg
@@ -948,6 +948,12 @@ VERNAC { tac2mode } EXTEND VernacLtac2
fun ~pstate -> Tac2entries.call ~pstate ~default t }
END
+GRAMMAR EXTEND Gram
+ GLOBAL: tac2mode;
+ tac2mode:
+ [ [ tac = G_vernac.query_command -> { tac None } ] ];
+END
+
{
open Stdarg