lean2/tests/lean/interactive/t5.lean

7 lines
126 B
Text
Raw Normal View History

Axiom magic (a : Bool) : a.
Theorem T (a : Bool) : a.
apply (** apply_tactic("magic") **).
done.
Show Environment 1.