lean2/tests/lean/run/tactic8.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

9 lines
195 B
Text

import logic
open tactic
theorem tst {A B : Prop} (H1 : A) (H2 : B) : A ∧ B ∧ A :=
by apply @and.intro;
apply (show A, from H1);
apply (show B ∧ A, from and.intro H2 H1)
check @tst