lean2/tests/lean/run/570.lean

17 lines
247 B
Text
Raw Permalink Normal View History

open nat
variables (P : → Prop)
example (H1 : ∃n, P n) : ∃n, P n :=
begin
cases H1 with n p,
apply (exists.intro n),
assumption
end
example (H1 : ∃n, P n) : ∃n, P n :=
begin
cases H1 with n p,
existsi n,
assumption
end