aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Notations.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-17 20:28:23 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-17 20:28:23 +0000
commit6b391cc61a35d1ef42f88d18f9c428c369180493 (patch)
treec402fcb05a8dd450dca2191607c11351633cfac0 /test-suite/success/Notations.v
parent9d7a9ab7c8182dff99d5afd078747f5d6b1247f0 (diff)
Fixed a notation bug when extending binder_constr with empty levels
(see Notations.v). Improved the "already occurs in a different scope" test and message. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12399 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/Notations.v')
-rw-r--r--test-suite/success/Notations.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/success/Notations.v b/test-suite/success/Notations.v
index 1bff74933..b09c6c9a7 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -43,3 +43,8 @@ Notation "'exists' x , P" := (x, P)
(at level 200, x ident, right associativity, only parsing).
Definition foo P := let '(exists x, Q) := P in x = Q :> nat.
+
+(* Check empty levels when extending binder_constr *)
+
+Notation "'exists' x >= y , P" := (exists x, x >= y /\ P)%nat
+ (at level 200, x ident, right associativity, y at level 69).