aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Notations.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-24 17:36:32 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-24 17:52:27 +0200
commit166634c57bbad2e727364a97bf30bc3d67d2f2a8 (patch)
treea0dfe52b0fa88c18f1a6cbfa5a4f57e5459dd5b1 /test-suite/success/Notations.v
parent71f69e26b595c2a403184cf805afaf9d46f8a0b3 (diff)
Merge branch 'v8.5' into v8.6
+ a few improvements on 5f1dd4c40 (lexing of { and }).
Diffstat (limited to 'test-suite/success/Notations.v')
-rw-r--r--test-suite/success/Notations.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/success/Notations.v b/test-suite/success/Notations.v
index 30abd961b..666c91257 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -115,3 +115,10 @@ Notation "[ a , .. , b ]" := (a, (.. (b,tt) ..)).
Require Import Coq.Vectors.VectorDef.
Import VectorNotations.
Goal True. idtac; []. (* important for test: no space here *) constructor. Qed.
+
+(* Check parsing of { and } is not affected by notations #3479 *)
+Notation " |- {{ a }} b" := (a=b) (no associativity, at level 10).
+Goal True.
+{{ exact I. }}
+Qed.
+Check |- {{ 0 }} 0.