lean2/tests/lean/run/tactic8.lean

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 B ∧ A, from and.intro H2 H1);
apply (show A, from H1)
check @tst