aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2021-03-25 15:02:51 +0100
committerPierre-Marie Pédrot2021-03-25 15:12:53 +0100
commit4a865fbce27d2b5ba0824ad52db0fea36ede0a9e (patch)
treec0ac404bee392afe92bbfab3403cb1ddf3d59b43 /test-suite/bugs
parentd328a04d5e533a8591dfb3f2fa3d0e0852037f33 (diff)
Fix the redeclaration check for Ltac2 entry points.
Fixes #14003: Ltac2 redefinition check is broken.
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/bug_14003.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/bug_14003.v b/test-suite/bugs/closed/bug_14003.v
new file mode 100644
index 0000000000..9e7055045d
--- /dev/null
+++ b/test-suite/bugs/closed/bug_14003.v
@@ -0,0 +1,19 @@
+Require Import Ltac2.Ltac2.
+
+Module Foo.
+
+Ltac2 foo := ().
+Ltac2 Type bar := [ BAR ].
+Ltac2 Type quz := [ .. ].
+Ltac2 Type quz ::= [ QUZ ].
+
+End Foo.
+
+Import Foo.
+
+(* Check that redeclaration checks are based on absolute names *)
+
+Ltac2 foo := ().
+Ltac2 Type bar := [ ].
+Ltac2 Type qux := [ BAR ].
+Ltac2 Type quz ::= [ QUZ ].