Skip to content
Snippets Groups Projects
Commit e7613555 authored by Ralf Jung's avatar Ralf Jung
Browse files

test tele_app notation

parent a03c40c5
No related branches found
No related tags found
1 merge request!342drop support for Coq 8.10
Pipeline #58315 passed
...@@ -18,3 +18,5 @@ ...@@ -18,3 +18,5 @@
Hγ : γ1 x Hγ : γ1 x
============================ ============================
γ1 x ∨ γ2 x γ1 x ∨ γ2 x
[TEST x y : nat, x = y]
: Prop
...@@ -31,3 +31,13 @@ Proof. ...@@ -31,3 +31,13 @@ Proof.
Qed. Qed.
End tests. End tests.
End accessor. End accessor.
(* Type inference for tele_app-based notation.
(Relies on [&] bidirectionality hint of tele_app.) *)
Definition test {TT : tele} (t : TT Prop) : Prop :=
.. x, t x t x.
Notation "'[TEST' x .. z , P ']'" :=
(test (TT:=(TeleS (fun x => .. (TeleS (fun z => TeleO)) ..)))
(tele_app (λ x, .. (λ z, P) ..)))
(x binder, z binder).
Check [TEST (x y : nat), x = y].
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment