lean2/tests/lean/run/tactic_notation.lean

12 lines
212 B
Text
Raw Normal View History

import logic
theorem tst1 (a b c : Prop) : a → b → a ∧ b :=
begin
intros,
apply and.intro,
assumption
end
theorem tst2 (a b c : Prop) : a → b → a ∧ b :=
by intros; apply and.intro; assumption