2015-02-04 23:30:18 +00:00
|
|
|
import data.nat
|
|
|
|
open algebra
|
|
|
|
|
|
|
|
theorem test {A : Type} [s : comm_ring A] (a b c : A) : a + b + c = a + c + b :=
|
|
|
|
begin
|
2015-02-05 04:16:24 +00:00
|
|
|
rewrite [add.assoc, {b + _}add.comm, -add.assoc]
|
2015-02-04 23:30:18 +00:00
|
|
|
end
|
|
|
|
|
2015-05-09 03:54:16 +00:00
|
|
|
reveal test
|
2015-02-04 23:30:18 +00:00
|
|
|
print definition test
|