aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Notations.v
diff options
context:
space:
mode:
authorGravatar Ralf Jung <post@ralfj.de>2017-02-14 12:36:15 +0100
committerGravatar Ralf Jung <post@ralfj.de>2017-02-16 16:47:12 +0100
commit8ce49dd1b436a17c4ee29c2893133829daac75f0 (patch)
treec5b53f5bf86ee07e53d43eec53099ba92ae19503 /test-suite/success/Notations.v
parent55cb913f029308e97bd262fc18d4338f404e7561 (diff)
reject notations that are both 'only printing' and 'only parsing'
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 32baeaa57..52acad746 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -132,3 +132,6 @@ Qed.
(* Check that we can have notations without any symbol iff they are "only printing". *)
Fail Notation "" := (@nil).
Notation "" := (@nil) (only printing).
+
+(* Check that a notation cannot be neither parsing nor printing. *)
+Fail Notation "'foobarkeyword'" := (@nil) (only parsing, only printing).