lean2/tests/lean/run/tactic1.lean

4 lines
78 B
Text

import logic
theorem tst {A B : Prop} (H1 : A) (H2 : B) : A
:= by assumption