Regular elements #
By definition, a regular element in a commutative ring is a non-zero divisor.
Lemma isRegular_of_ne_zero
implies that every non-zero element of an integral domain is regular.
Since it assumes that the ring is a CancelMonoidWithZero
it applies also, for instance, to ℕ
.
The lemmas in Section MulZeroClass
show that the 0
element is (left/right-)regular if and
only if the MulZeroClass
is trivial. This is useful when figuring out stopping conditions for
regular sequences: if 0
is ever an element of a regular sequence, then we can extend the sequence
by adding one further 0
.
The final goal is to develop part of the API to prove, eventually, results about non-zero-divisors.
In a semigroup, the product of left-regular elements is left-regular.
In an additive semigroup, the sum of add-left-regular elements is add-left.regular.
In a semigroup, the product of right-regular elements is right-regular.
In an additive semigroup, the sum of add-right-regular elements is add-right-regular.
In an additive semigroup, the sum of add-regular elements is add-regular.
If an element b
becomes left-regular after multiplying it on the left by a left-regular
element, then b
is left-regular.
If an element b
becomes add-left-regular after adding to it on the left
an add-left-regular element, then b
is add-left-regular.
An element is left-regular if and only if multiplying it on the left by a left-regular element is left-regular.
An element is add-left-regular if and only if adding to it on the left an add-left-regular element is add-left-regular.
If an element b
becomes right-regular after multiplying it on the right by a right-regular
element, then b
is right-regular.
If an element b
becomes add-right-regular after adding to it on the right
an add-right-regular element, then b
is add-right-regular.
An element is right-regular if and only if multiplying it on the right with a right-regular element is right-regular.
An element is add-right-regular if and only if adding it on the right to an add-right-regular element is add-right-regular.
Two elements a
and b
are add-regular if and only if both sums a + b
and
b + a
are add-regular.
The "most used" implication of add_and_add_iff
, with split
hypotheses, instead of ∧
.
If multiplying by 1
on either side is the identity, 1
is regular.
If adding 0
on either side is the identity, 0
is regular.
A product is regular if and only if the factors are.
A sum is add-regular if and only if the summands are.
An element admitting a left inverse is left-regular.
An element admitting a left additive opposite is add-left-regular.
An element admitting a right inverse is right-regular.
An element admitting a right additive opposite is add-right-regular.
If R
is an additive monoid, an element in add_units R
is add-regular.
An additive unit in an additive monoid is add-regular.
Any power of a left-regular element is left-regular.
Any power of a right-regular element is right-regular.
An element a
is left-regular if and only if a positive power of a
is left-regular.
An element a
is right-regular if and only if a positive power of a
is right-regular.