c50227ea6e
This commit also adds the tactic rapply that corresponds to the previous semantics we have been using.
9 lines
195 B
Text
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
|