lean2/tests/lean/empty_thm.lean
Leonardo de Moura 368f9d347e refactor(frontends/lean): approach used to parse tactics
The previous approach was too fragile

TODO: we should add separate parsing tables for tactics
2015-03-05 18:11:21 -08:00

10 lines
158 B
Text

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