aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Notations2.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-19 19:13:23 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-19 19:40:13 +0200
commit75a48bfc6b91f1e5095d9cdfbcc0ae2bf8cf16ec (patch)
tree3954479b911b7681255764be0bcb13d72f52e8bd /test-suite/output/Notations2.v
parentb038ff00e3d1873bed580c13df1b18ce0510abb2 (diff)
Fixing #4677 (collision of a global variable and of a local variable
while eta-expanding a notation) + a more serious variant of it (alpha-conversion incorrect wrt eta-expansion).
Diffstat (limited to 'test-suite/output/Notations2.v')
-rw-r--r--test-suite/output/Notations2.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/output/Notations2.v b/test-suite/output/Notations2.v
index e53c94ef0..c9efe1ead 100644
--- a/test-suite/output/Notations2.v
+++ b/test-suite/output/Notations2.v
@@ -68,8 +68,10 @@ Check let' f x y (a:=0) z (b:bool) := x+y+z+1 in f 0 1 2.
(* In practice, only the printing rule is used here *)
(* Note: does not work for pattern *)
+Module A.
Notation "f ( x )" := (f x) (at level 10, format "f ( x )").
Check fun f x => f x + S x.
+End A.
Open Scope list_scope.
Notation list1 := (1::nil)%list.
@@ -98,3 +100,9 @@ Notation "# x : T => t" := (fun x : T => t)
Check # x : nat => x.
Check # _ : nat => 2.
+
+(* Check bug 4677 *)
+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).