lean2/tests/lean/empty_thm.lean
Leonardo de Moura 05b0f24cb5 fix(frontends/lean/decl_cmds): improve error message for invalid end of theorem
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-08-17 17:03:54 -07:00

10 lines
165 B
Text

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