2015-02-22 18:20:27 -08:00
|
|
|
import algebra.group
|
|
|
|
open algebra
|
|
|
|
|
2015-04-21 19:33:21 -07:00
|
|
|
section
|
2015-02-22 18:20:27 -08:00
|
|
|
variable {A : Type}
|
|
|
|
variable [s : comm_monoid A]
|
|
|
|
include s
|
|
|
|
|
2015-05-18 15:45:23 -07:00
|
|
|
theorem one_mul_one : 1 * 1 = (1:A) :=
|
2015-02-22 18:20:27 -08:00
|
|
|
mul_one 1
|
|
|
|
end
|
|
|
|
|
2015-04-21 19:33:21 -07:00
|
|
|
section
|
2015-02-22 18:20:27 -08:00
|
|
|
variable {A : Type}
|
|
|
|
variable [s : comm_group A]
|
|
|
|
include s
|
|
|
|
|
2015-10-13 15:39:03 -07:00
|
|
|
theorem one_mul_one2 : (one : A) * 1 = 1 :=
|
2015-02-22 18:20:27 -08:00
|
|
|
by rewrite one_mul_one
|
|
|
|
end
|