lean2/tests/lean/run/using_expr.lean
2015-04-04 15:25:07 -07:00

8 lines
209 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, assumption
end