Documentation

Mathlib.Algebra.Regular.Defs

Regular elements #

We introduce left-regular, right-regular and regular elements, along with their to_additive analogues add-left-regular, add-right-regular and add-regular elements.

For monoids where every element is regular, see IsCancelMul and nearby typeclasses.

def IsLeftRegular {R : Type u_1} [Mul R] (c : R) :

A left-regular element is an element c such that multiplication on the left by c is injective.

Equations
Instances For
    def IsAddLeftRegular {R : Type u_1} [Add R] (c : R) :

    An add-left-regular element is an element c such that addition on the left by c is injective.

    Equations
    Instances For
      def IsRightRegular {R : Type u_1} [Mul R] (c : R) :

      A right-regular element is an element c such that multiplication on the right by c is injective.

      Equations
      Instances For
        def IsAddRightRegular {R : Type u_1} [Add R] (c : R) :

        An add-right-regular element is an element c such that addition on the right by c is injective.

        Equations
        Instances For
          structure IsAddRegular {R : Type u_2} [Add R] (c : R) :

          An add-regular element is an element c such that addition by c both on the left and on the right is injective.

          Instances For
            structure IsRegular {R : Type u_1} [Mul R] (c : R) :

            A regular element is an element c such that multiplication by c both on the left and on the right is injective.

            Instances For