lean2/tests/lean/run/tactic3.lean

10 lines
193 B
Text
Raw Normal View History

import logic
open tactic
theorem tst {A B : Prop} (H1 : A) (H2 : B) : A
:= by (trace "first"; state; now |
trace "second"; state; fail |
trace "third"; assumption)
check tst