lean2/tests/lean/run/rewriter1.lean
2015-02-04 15:30:18 -08:00

9 lines
192 B
Text

import data.nat
open algebra
theorem test {A : Type} [s : comm_ring A] (a b c : A) : a + b + c = a + c + b :=
begin
rewrite add.assoc [b + _]add.comm -add.assoc,
end
print definition test