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-10-12 16:07:56 +0200
commit5dd690ee5975262d34d8dcc44191138c8d326f65 (patch)
treec54f5fb3f8cfee72b8ee640bff2df37957b921d2 /test-suite/success/Notations.v
parentd48176857632e1d2a0af0a31dc922f3c52047707 (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) ..)).