aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorcoqbot-app[bot]2021-04-16 15:54:04 +0000
committerGitHub2021-04-16 15:54:04 +0000
commitf337187f0ac4c2062031225234fd23b436b979b5 (patch)
tree8e367c5a3ea632487a1c805b04aa593c77225b1a /test-suite
parentfaafe565b942736acc940c8374914fe0284b0b3d (diff)
parent650461653aa1d4bc47509f0a2c49c3a235fb6381 (diff)
Merge PR #13939: Allow scope delimiters in Ltac2 open_constr:(...) quotation.
Reviewed-by: JasonGross
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/bug_12806.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/bug_12806.v b/test-suite/bugs/closed/bug_12806.v
new file mode 100644
index 0000000000..ee221d33a6
--- /dev/null
+++ b/test-suite/bugs/closed/bug_12806.v
@@ -0,0 +1,9 @@
+Require Import Ltac2.Ltac2.
+
+Declare Scope my_scope.
+Delimit Scope my_scope with my_scope.
+
+Notation "###" := tt : my_scope.
+
+Ltac2 Notation "bar" c(open_constr(my_scope)) := c.
+Ltac2 Eval bar ###.