aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Notations2.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-09-12 17:22:03 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-09-12 17:22:03 +0200
commit90e5945e1666540bc18e7a9b831d136041f4e487 (patch)
tree9af1cee10f24c6114c196ba4e1302b2931899f7d /test-suite/output/Notations2.v
parent74f8381ed943f1e786b32c49fb31f14fd488dc9c (diff)
Fixing a recursive notation bug raised on coq-club on Sep 12, 2016.
Diffstat (limited to 'test-suite/output/Notations2.v')
-rw-r--r--test-suite/output/Notations2.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/output/Notations2.v b/test-suite/output/Notations2.v
index 4e0d135d7..3f3945052 100644
--- a/test-suite/output/Notations2.v
+++ b/test-suite/output/Notations2.v
@@ -106,3 +106,8 @@ Check fun x (H:le x 0) => exist (le x) 0 H.
Parameters (A : Set) (x y : A) (Q : A -> A -> Prop) (conj : Q x y).
Check (exist (Q x) y conj).
+
+(* Check bug raised on coq-club on Sep 12, 2016 *)
+
+Notation "{ x , y , .. , v }" := (fun a => (or .. (or (a = x) (a = y)) .. (a = v))).
+Check ({1, 2}).