Semirings and rings #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file gives lemmas about semirings, rings and domains.
This is analogous to algebra.group.basic
,
the difference being that the former is about +
and *
separately, while
the present file is about their interaction.
For the definitions of semirings and rings see algebra.ring.defs
.
theorem
commute.mul_self_eq_mul_self_iff
{R : Type x}
[non_unital_non_assoc_ring R]
[no_zero_divisors R]
{a b : R}
(h : commute a b) :
@[simp]
@[simp]
@[simp]
theorem
commute.neg_one_right
{R : Type x}
[mul_one_class R]
[has_distrib_neg R]
(a : R) :
commute a (-1)
@[simp]
theorem
commute.neg_one_left
{R : Type x}
[mul_one_class R]
[has_distrib_neg R]
(a : R) :
commute (-1) a
@[simp]
@[simp]