lean2/tests/lean/run/rewriter6.lean

14 lines
357 B
Text
Raw Normal View History

import data.int
open int
theorem abs_thm1 (a b : int) : a - b = a + -b :=
by rewrite ↑sub -- unfold sub
theorem abs_thm2 (a b : int) : a - b = a + -b :=
by rewrite ^sub -- unfold sub
definition double (x : int) := x + x
theorem double_zero (x : int) : double (0 + x) = (1 + 1)*x :=
2015-10-23 14:24:30 +00:00
by rewrite [↑double, int.zero_add, int.right_distrib, int.one_mul]