lean2/tests/lean/run/454.lean

7 lines
148 B
Text
Raw Normal View History

constants (A : Type₁) (P : A → Type₁) (H : Π{a b : A}, P a → P b) (a b : A) (K : P a)
theorem foo : P b :=
begin
apply H, {apply K}
end