Documentation

Mathlib.Algebra.Ring.Center

Centers of rings #

@[simp]
theorem Set.natCast_mem_center (M : Type u_1) [NonAssocSemiring M] (n : ) :
n center M
@[simp]
theorem Set.ofNat_mem_center (M : Type u_1) [NonAssocSemiring M] (n : ) [n.AtLeastTwo] :
@[simp]
theorem Set.intCast_mem_center (M : Type u_1) [NonAssocRing M] (n : ) :
n center M
@[simp]
theorem Set.add_mem_center {M : Type u_1} [Distrib M] {a b : M} (ha : a center M) (hb : b center M) :
a + b center M
@[simp]
theorem Set.neg_mem_center {M : Type u_1} [NonUnitalNonAssocRing M] {a : M} (ha : a center M) :