Documentation

Mathlib.Algebra.Order.Ring.Idempotent

Boolean algebra structure on idempotents in a commutative (semi)ring #

We show that the idempotent in a commutative ring form a Boolean algebra, with complement given by a ↦ 1 - a and infimum given by multiplication. In a commutative semiring where subtraction is not available, it is still true that pairs of elements (a, b) satisfying a * b = 0 and a + b = 1 form a Boolean algebra (such elements are automatically idempotents, and such a pair is uniquely determined by either a or b).

instance instHasComplSubtypeProdAndEqHMulFstSndOfNatHAdd {R : Type u_1} [CommMonoid R] [AddCommMonoid R] :
HasCompl { a : R × R // a.1 * a.2 = 0 a.1 + a.2 = 1 }
Equations
theorem eq_of_mul_eq_add_eq_one {R : Type u_1} [NonAssocSemiring R] (a : R) {b c : R} (mul : a * b = c * a) (add_ab : a + b = 1) (add_ac : a + c = 1) :
b = c
theorem mul_eq_zero_add_eq_one_ext_left {R : Type u_1} [CommSemiring R] {a b : { a : R × R // a.1 * a.2 = 0 a.1 + a.2 = 1 }} (eq : (↑a).1 = (↑b).1) :
a = b
theorem mul_eq_zero_add_eq_one_ext_right {R : Type u_1} [CommSemiring R] {a b : { a : R × R // a.1 * a.2 = 0 a.1 + a.2 = 1 }} (eq : (↑a).2 = (↑b).2) :
a = b
instance instPartialOrderSubtypeProdAndEqHMulFstSndOfNatHAdd {R : Type u_1} [CommSemiring R] :
PartialOrder { a : R × R // a.1 * a.2 = 0 a.1 + a.2 = 1 }
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
def OrderIso.isIdempotentElemMulZeroAddOne {R : Type u_1} [CommRing R] :
{ a : R // IsIdempotentElem a } ≃o { a : R × R // a.1 * a.2 = 0 a.1 + a.2 = 1 }

In a commutative ring, the idempotents are in 1-1 correspondence with pairs of elements whose product is 0 and whose sum is 1. The correspondence is given by a ↔ (a, 1 - a).

Equations
  • One or more equations did not get rendered due to their size.
Instances For