e379034b95
- It uses the unifier in "conservative" mode - It only affects the current goal closes #570
16 lines
247 B
Text
16 lines
247 B
Text
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
|