e379034b95
- It uses the unifier in "conservative" mode - It only affects the current goal closes #570
8 lines
216 B
Text
8 lines
216 B
Text
example (p q : Prop) (H : p ∧ q) : p ∧ q ∧ p :=
|
|
have Hp : p, from and.elim_left H,
|
|
have Hq : q, from and.elim_right H,
|
|
using Hp Hq,
|
|
begin
|
|
apply and.intro, assumption,
|
|
apply and.intro, repeat assumption
|
|
end
|