aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-08-13 20:05:03 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-02-20 10:03:04 +0100
commitd4c2ed95fcfd64cdcc10e51e40be739d9f1c4a74 (patch)
tree4843bf72c79905f811d6f3f5ac4cdd4d81943e65 /test-suite/output
parent7c10b4020e061fb14e01cb3abc92bb5265aa65b9 (diff)
Allows recursive patterns for binders to be associative on the left.
This makes treatment of recursive binders closer to the one of recursive terms. It is unclear whether there are interesting notations liable to use this, but this shall make easier mixing recursive binders and recursive terms as in next commits. Example of (artificial) notation that this commit supports: Notation "! x .. y # A #" := (.. (A,(forall x, True)) ..,(forall y, True)) (at level 200, x binder).
Diffstat (limited to 'test-suite/output')
-rw-r--r--test-suite/output/Notations3.out2
-rw-r--r--test-suite/output/Notations3.v4
2 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/output/Notations3.out b/test-suite/output/Notations3.out
index cf69874ca..e114ea894 100644
--- a/test-suite/output/Notations3.out
+++ b/test-suite/output/Notations3.out
@@ -161,3 +161,5 @@ exists_true (A : Type) (R : A -> A -> Prop) (_ : Reflexive R),
exists_true (x : nat) (A : Type) (R : A -> A -> Prop)
(_ : Reflexive R) (y : nat), x + y = 0 -> forall z : A, R z z
: Prop
+{{{{True, nat -> True}}, nat -> True}}
+ : Prop * Prop * Prop
diff --git a/test-suite/output/Notations3.v b/test-suite/output/Notations3.v
index 3e07fbce9..a7fed3561 100644
--- a/test-suite/output/Notations3.v
+++ b/test-suite/output/Notations3.v
@@ -278,3 +278,7 @@ Class Reflexive {A:Type} (R : A->A->Prop) := reflexivity : forall x : A, R x x.
Check exists_true `{Reflexive A R}, forall x, R x x.
Check exists_true x `{Reflexive A R} y, x+y=0 -> forall z, R z z.
End G.
+
+(* Allows recursive patterns for binders to be associative on the left *)
+Notation "!! x .. y # A #" := (.. (A,(forall x, True)) ..,(forall y, True)) (at level 200, x binder).
+Check !! a b : nat # True #.