lean2/tests/lean/simp_tac.lean
Leonardo de Moura 4d25cb7f47 feat(library/tactic): add simplify_tactic based on the simplifier
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-26 18:53:18 -08:00

8 lines
286 B
Text

import tactic
-- Create a simple rewrite set
rewrite_set simple
add_rewrite Nat::add_zeror Nat::add_zerol Nat::add_comm eq_id : simple
-- Prove the following theorem using the simplifier with the rewrite set simple
theorem Test (a b : Nat) : 0 + a + 0 + b = b + a := (by simp simple)