This repository was archived by the owner on Jul 24, 2024. It is now read-only.
File tree Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -13,8 +13,8 @@ import algebra.iterate_hom
13
13
We introduce left-regular, right-regular and regular elements.
14
14
15
15
By definition, a regular element in a commutative ring is a non-zero divisor.
16
- Lemma `is_regular_of_cancel_monoid_with_zero ` implies that every non-zero element of an integral
17
- domain is regular .
16
+ Lemma `is_regular_of_ne_zero ` implies that every non-zero element of an integral domain is regular.
17
+ Since it assumes that the ring is a `cancel_monoid_with_zero` it applies also, for instance, to `ℕ` .
18
18
19
19
The lemmas in Section `mul_zero_class` show that the `0` element is (left/right-)regular if and
20
20
only if the `mul_zero_class` is trivial. This is useful when figuring out stopping conditions for
@@ -279,7 +279,7 @@ section cancel_monoid_with_zero
279
279
variables [cancel_monoid_with_zero R]
280
280
281
281
/-- Non-zero elements of an integral domain are regular. -/
282
- lemma is_regular_of_cancel_monoid_with_zero (a0 : a ≠ 0 ) : is_regular a :=
282
+ lemma is_regular_of_ne_zero (a0 : a ≠ 0 ) : is_regular a :=
283
283
⟨λ b c, (mul_right_inj' a0).mp, λ b c, (mul_left_inj' a0).mp⟩
284
284
285
285
end cancel_monoid_with_zero
You can’t perform that action at this time.
0 commit comments