0a67679afb
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
18 lines
616 B
Text
18 lines
616 B
Text
Set pp::colors false
|
|
Variable f : Pi (A : Type), A -> Bool
|
|
Show fun (A B : Type) (a : _), f B a
|
|
(* The following one should produce an error *)
|
|
Show fun (A : Type) (a : _) (B : Type), f B a
|
|
|
|
Variable myeq : Pi (A : Type U), A -> A -> Bool
|
|
Show myeq _ (fun (A : Type) (a : _), a) (fun (B : Type) (b : B), b)
|
|
Check myeq _ (fun (A : Type) (a : _), a) (fun (B : Type) (b : B), b)
|
|
|
|
|
|
Variable R : Type -> Bool
|
|
Variable h : (Pi (A : Type), R A) -> Bool
|
|
Check (fun (H : Bool)
|
|
(f1 : Pi (A : Type), R _)
|
|
(g1 : Pi (A : Type), R A)
|
|
(G : Pi (A : Type), myeq _ (f1 _) (g1 A)),
|
|
h f1)
|