aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Notations.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-12-18 22:11:29 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-12-18 22:11:29 +0000
commit6d7ee3b6267ef0d5bd3367d9230d9a4849aa42aa (patch)
tree9b51e58f2645b64afd1462ead83c460b873b7965 /test-suite/success/Notations.v
parentd8cc0ec7d99cc5f26b432b6ded95467064456ebf (diff)
Fixing bug #2634 (unscoped notations were disturbing the
interpretation order of scoped notations). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14819 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/Notations.v')
-rw-r--r--test-suite/success/Notations.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/success/Notations.v b/test-suite/success/Notations.v
index ddad217b3..f5f5a9d14 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -75,3 +75,14 @@ End B.
(* Should succeed *)
Definition n := 5 * 5.
+
+(* Check that lonely notations (here FOO) do not modify the visibility
+ of scoped interpretations (bug #2634 fixed in r14819) *)
+
+Notation "x ++++ y" := (mult x y) (at level 40).
+Notation "x ++++ y" := (plus x y) : A_scope.
+Open Scope A_scope.
+Notation "'FOO' x" := (S x) (at level 40).
+Goal (2 ++++ 3) = 5.
+reflexivity.
+Abort.