lean2/tests/lean/show_tac.lean
Leonardo de Moura c133d26505 feat(frontends/lean/builtin_exprs): change how 'show' is processed in tactics
Unresolved placeholders were not being reported
2015-05-19 16:23:50 -07:00

7 lines
185 B
Text

example (a b : Prop) : a ∧ b → b ∧ a :=
begin
intro Hab,
have Ha : a, from and.elim_left Hab,
have Hb : b, from and.elim_right Hab,
show b ∧ a, from and.intro _ Ha
end