lean2/tests/lean/empty_thm.lean
Leonardo de Moura e51c4ad2e9 feat(frontends/lean): rename 'using' command to 'open'
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-09-03 16:00:38 -07:00

10 lines
164 B
Text

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