summaryrefslogtreecommitdiff
path: root/test-suite/success/Notations.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/Notations.v')
-rw-r--r--test-suite/success/Notations.v16
1 files changed, 15 insertions, 1 deletions
diff --git a/test-suite/success/Notations.v b/test-suite/success/Notations.v
index a9e2c59a..facd5509 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -1,5 +1,5 @@
(* Check that "where" clause behaves as if given independently of the *)
-(* definition (variant of bug #113? submitted by Assia Mahboubi) *)
+(* definition (variant of bug #1132 submitted by Assia Mahboubi) *)
Fixpoint plus1 (n m:nat) {struct n} : nat :=
match n with
@@ -7,3 +7,17 @@ Fixpoint plus1 (n m:nat) {struct n} : nat :=
| S p => S (p+m)
end
where "n + m" := (plus1 n m) : nat_scope.
+
+(* Check behaviour wrt yet empty levels (see Stephane's bug #1850) *)
+
+Parameter P : Type -> Type -> Type -> Type.
+Notation "e |= t --> v" := (P e t v) (at level 100, t at level 54).
+Check (nat |= nat --> nat).
+
+(* Check that first non empty definition at an empty level can be of any
+ associativity *)
+
+Definition marker := O.
+Notation "x +1" := (S x) (at level 8, left associativity).
+Reset marker.
+Notation "x +1" := (S x) (at level 8, right associativity).