lean2/examples/lean/ex4.lean
Leonardo de Moura 028a9bd9bd feat(frontends/lean/scanner): use Lua style comments in Lean
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-05 08:53:27 -08:00

8 lines
239 B
Text

Import Int
Import tactic
Definition a : Nat := 10
-- Trivial indicates a "proof by evaluation"
Theorem T1 : a > 0 := Trivial
Theorem T2 : a - 5 > 3 := Trivial
-- The next one is commented because it fails
-- Theorem T3 : a > 11 := Trivial