lean2/tests/lean/empty_thm.lean

11 lines
165 B
Text
Raw Normal View History

import logic tools.tactic
using tactic
definition simple := apply trivial
tactic_hint simple
theorem foo : true
theorem foo2 (a : Prop) : a :
theorem foo3 : true