aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-03-17 09:12:38 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-03-17 09:12:38 +0100
commitdbbc4da0e52567325d74128dccd1b54760cb970d (patch)
tree1c10abf7767d04929229818018accdf33eb8b0f2 /test-suite
parent037b21fc9913958d9e38866cf014fcec0ef78311 (diff)
parent8ce49dd1b436a17c4ee29c2893133829daac75f0 (diff)
Merge PR#429: Don't require printing-only notation to be productive
Diffstat (limited to 'test-suite')
-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 07bbb60c4..52acad746 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -128,3 +128,10 @@ Notation " |- {{ a }} b" := (a=b) (no associativity, at level 10).
Goal True.
{{ exact I. }}
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).