aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Notations3.out
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-05-20 21:27:34 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-05-31 00:35:46 +0200
commit9ee5808746cbcf6e04c08e6a2e798b6cbb34bb06 (patch)
tree4304ee584c02cbee626dc1ace75e384faf990e4a /test-suite/output/Notations3.out
parentbcc9165aec1a80d563d7060ef127ad022e9ed008 (diff)
Fixing a too lax constraint for finding recursive binder part of a notation.
This was preventing to work examples such as: Notation "[ x ; .. ; y ; z ]" := ((x,((fun u => u), .. (y,(fun u =>u,z)) ..))).
Diffstat (limited to 'test-suite/output/Notations3.out')
-rw-r--r--test-suite/output/Notations3.out5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/output/Notations3.out b/test-suite/output/Notations3.out
index 4d59a92cb..f4ecfd736 100644
--- a/test-suite/output/Notations3.out
+++ b/test-suite/output/Notations3.out
@@ -98,5 +98,10 @@ fun n : nat => foo4 n (fun _ y : nat => ETA z : nat, (fun _ : nat => y = 0))
: nat -> Prop
tele (t : Type) '(y, z) (x : t0) := tt
: forall t : Type, nat * nat -> t -> fpack
+[fun x : nat => x + 0;; fun x : nat => x + 1;; fun x : nat => x + 2]
+ : (nat -> nat) *
+ ((nat -> nat) *
+ ((nat -> nat) *
+ ((nat -> nat) * ((nat -> nat) * ((nat -> nat) * (nat -> nat))))))
foo5 x nat x
: nat -> nat