aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Notations.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-08-12 13:32:05 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-09-12 20:27:14 +0200
commita267b06c4a237ce3e4ce257e47f6429543804baa (patch)
treef8e84c33cbf8935d19c3e167bb4dbf9cd52e6a16 /test-suite/success/Notations.v
parentcc94172036789cfef28007f59510b7f17df5d45d (diff)
Fixing little inaccuracy in coercions to ident or name.
For instance, we don't want "id@{u}" to be coerced to id, or "?[n]" to "_".
Diffstat (limited to 'test-suite/success/Notations.v')
-rw-r--r--test-suite/success/Notations.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/success/Notations.v b/test-suite/success/Notations.v
index 837f2efd0..4d04f2cf9 100644
--- a/test-suite/success/Notations.v
+++ b/test-suite/success/Notations.v
@@ -142,3 +142,8 @@ Fail Notation "'foobarkeyword'" := (@nil) (only parsing, only printing).
Reserved Notation "x === y" (at level 50).
Inductive EQ {A} (x:A) : A -> Prop := REFL : x === x
where "x === y" := (EQ x y).
+
+(* Check that strictly ident or _ are coerced to a name *)
+
+Fail Check {x@{u},y|x=x}.
+Fail Check {?[n],y|0=0}.