aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_3468.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/bug_3468.v')
-rw-r--r--test-suite/bugs/closed/bug_3468.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/bug_3468.v b/test-suite/bugs/closed/bug_3468.v
index 6ff394bca6..8d7d97d7aa 100644
--- a/test-suite/bugs/closed/bug_3468.v
+++ b/test-suite/bugs/closed/bug_3468.v
@@ -26,4 +26,5 @@ Notation "& b" := ltac:(exact (b)%my) (at level 100, only parsing): my_scope.
Definition test := (& (@4))%my.
(* Check inconsistent scopes *)
+Set Warnings "+inconsistent-scopes".
Fail Notation bar3 a := (let __ := ltac:(exact a%nat) in a%bool) (only parsing).