mathlib3 documentation

algebra.ring.regular

Lemmas about regular elements in rings. #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

theorem is_left_regular_of_non_zero_divisor {α : Type u_1} [non_unital_non_assoc_ring α] (k : α) (h : (x : α), k * x = 0 x = 0) :

Left mul by a k : α over [ring α] is injective, if k is not a zero divisor. The typeclass that restricts all terms of α to have this property is no_zero_divisors.

theorem is_right_regular_of_non_zero_divisor {α : Type u_1} [non_unital_non_assoc_ring α] (k : α) (h : (x : α), x * k = 0 x = 0) :

Right mul by a k : α over [ring α] is injective, if k is not a zero divisor. The typeclass that restricts all terms of α to have this property is no_zero_divisors.

theorem is_regular_of_ne_zero' {α : Type u_1} [non_unital_non_assoc_ring α] [no_zero_divisors α] {k : α} (hk : k 0) :