2015-05-03 02:33:59 +00:00
|
|
|
inductive foo {A : Type} : A → Type :=
|
|
|
|
mk : Π a : A, foo a
|
|
|
|
|
|
|
|
example (A : Type) (B : A → Type) (a : A) (H : foo a) (Hb : B a) : A :=
|
|
|
|
begin
|
|
|
|
cases H,
|
|
|
|
state,
|
|
|
|
assumption
|
|
|
|
end
|
|
|
|
|
|
|
|
inductive foo₂ {A : Type} : A → A → Type :=
|
|
|
|
mk : Π a b : A, foo₂ a b
|
|
|
|
|
|
|
|
example (A : Type) (B : A → Type) (f : A → A) (a : A) (H : foo₂ (f a) a) (Hb : H = H) (Hc : a = a) : A :=
|
|
|
|
begin
|
2015-05-14 21:32:54 +00:00
|
|
|
cases H,
|
2015-05-03 02:33:59 +00:00
|
|
|
state,
|
2015-05-14 21:32:54 +00:00
|
|
|
exact a
|
2015-05-03 02:33:59 +00:00
|
|
|
end
|