lean2/tests/lean/run/using_expr.lean
Leonardo de Moura e379034b95 feat(library/tactic): improve 'assumption' tactic
- It uses the unifier in "conservative" mode
- It only affects the current goal

closes #570
2015-05-02 17:33:54 -07:00

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