2014-01-08 08:38:39 +00:00
|
|
|
variable f : forall (A : Type), A -> Bool
|
2014-01-05 19:03:35 +00:00
|
|
|
print fun (A B : Type) (a : _), f B a
|
2014-01-05 16:52:46 +00:00
|
|
|
-- The following one should produce an error
|
2014-01-05 19:03:35 +00:00
|
|
|
print fun (A : Type) (a : _) (B : Type), f B a
|
2013-08-31 21:25:27 +00:00
|
|
|
|
2014-01-08 08:38:39 +00:00
|
|
|
variable myeq : forall A : (Type U), A -> A -> Bool
|
2014-01-05 19:03:35 +00:00
|
|
|
print myeq _ (fun (A : Type) (a : _), a) (fun (B : Type) (b : B), b)
|
2014-01-05 20:05:08 +00:00
|
|
|
check myeq _ (fun (A : Type) (a : _), a) (fun (B : Type) (b : B), b)
|
2013-08-31 21:25:27 +00:00
|
|
|
|
|
|
|
|
2014-01-05 20:05:08 +00:00
|
|
|
variable R : Type -> Bool
|
2014-01-08 08:38:39 +00:00
|
|
|
variable h : (forall (A : Type), R A) -> Bool
|
2014-01-05 20:05:08 +00:00
|
|
|
check (fun (H : Bool)
|
2014-01-08 08:38:39 +00:00
|
|
|
(f1 : forall (A : Type), R _)
|
|
|
|
(g1 : forall (A : Type), R A)
|
|
|
|
(G : forall (A : Type), myeq _ (f1 _) (g1 A)),
|
2013-08-31 21:25:27 +00:00
|
|
|
h f1)
|