aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-08-17 12:35:56 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-02-20 10:03:06 +0100
commit3a6b1d2c04ceeb568accbc9ddfc3fc0f14faf25b (patch)
tree52d6f018753666991104a6a63558b1ecef387bb8 /test-suite/output
parent149997b59c6711c551490c4e7601eaac59f5f675 (diff)
Respecting the ident/pattern distinction in notation modifiers.
Diffstat (limited to 'test-suite/output')
-rw-r--r--test-suite/output/Notations3.out3
-rw-r--r--test-suite/output/Notations3.v7
2 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/output/Notations3.out b/test-suite/output/Notations3.out
index fb2d375c2..7c47c0885 100644
--- a/test-suite/output/Notations3.out
+++ b/test-suite/output/Notations3.out
@@ -197,3 +197,6 @@ fun x : nat => if x is n .+ 1 then n else 1
: Set
exists2' {{x, y}}, x = 0 & y = 0
: Prop
+exists2 x : nat * nat,
+ let '{{y, z}} := x in y > z & let '{{y, z}} := x in z > y
+ : Prop
diff --git a/test-suite/output/Notations3.v b/test-suite/output/Notations3.v
index 46e0c1b1b..ee6f0a09e 100644
--- a/test-suite/output/Notations3.v
+++ b/test-suite/output/Notations3.v
@@ -338,9 +338,16 @@ Check fun x => if x is n.+1 then n else 1.
Check {(x,y)|x+y=0}.
+Module D.
Notation "'exists2'' x , p & q" := (ex2 (fun x => p) (fun x => q))
(at level 200, x pattern, p at level 200, right associativity,
format "'[' 'exists2'' '/ ' x , '/ ' '[' p & '/' q ']' ']'")
: type_scope.
Check exists2' (x,y), x=0 & y=0.
+End D.
+
+(* Ensuring for reparsability that printer of notations does not use a
+ pattern where only an ident could be reparsed *)
+
+Check ex2 (fun x => let '(y,z) := x in y>z) (fun x => let '(y,z) := x in z>y).