lean2/tests/lean/run/intros.lean
Leonardo de Moura c50227ea6e feat(library/tactic): change apply tactic semantics: goals are not reversed; and dependent arguments are not included
This commit also adds the tactic rapply that corresponds to the previous
semantics we have been using.
2014-10-22 18:11:09 -07:00

33 lines
596 B
Text

import logic tools.tactic
open tactic
theorem tst1 (a b : Prop) : a → b → b :=
by intro Ha; intro Hb; apply Hb
theorem tst2 (a b : Prop) : a → b → a ∧ b :=
by intro Ha; intro Hb; rapply and.intro; apply Hb; apply Ha
theorem tst3 (a b : Prop) : a → b → a ∧ b :=
begin
intro Ha,
intro Hb,
apply and.intro,
apply Ha,
apply Hb,
end
theorem tst4 (a b : Prop) : a → b → a ∧ b :=
begin
intros (Ha, Hb),
rapply and.intro,
apply Hb,
apply Ha
end
theorem tst5 (a b : Prop) : a → b → a ∧ b :=
begin
intros,
apply and.intro,
eassumption,
eassumption
end