aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Notations.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-07-16 16:24:59 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-07-16 16:24:59 +0200
commitf64a49297d90851780d453ce12f57ed4d4174438 (patch)
treee1c99575cf8c38253512edf4374bb3f4408d5b7f /test-suite/success/Notations.v
parent45250332a1e65d434432940a468312f2ab18a2e8 (diff)
Fixing a collision about the meta-variable ".." in recursive notations.
This happens when recursive notations are used to define recursive notations.
Diffstat (limited to 'test-suite/success/Notations.v')
-rw-r--r--test-suite/success/Notations.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/test-suite/success/Notations.v b/test-suite/success/Notations.v
index b72a06740..2f7c62972 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -107,3 +107,6 @@ Notation traverse_var f l := (traverse (fun l => f l) l).
Notation "'intros' x" := (S x) (at level 0).
Goal True -> True. intros H. exact H. Qed.
+
+(* Check absence of collision on ".." in nested notations with ".." *)
+Notation "[ a , .. , b ]" := (a, (.. (b,tt) ..)).