aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-03-22 14:33:22 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-03-22 14:36:14 +0100
commit8b73fd7c6ce423f8c8a2594e90200f2407795d52 (patch)
tree91db0f56763e6512016055a8dc47185f7317fe6b /test-suite/success
parent6e0ca299c407125a8d65f54ab424bdae3667125e (diff)
parentcd87eac3757d8925ff4ba7dee85efadb195153a3 (diff)
Merge branch 'v8.6'
Diffstat (limited to 'test-suite/success')
-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).