Documentation

Mathlib.Algebra.GroupWithZero.Units.Equiv

Multiplication by a nonzero element in a GroupWithZero is a permutation. #

def Equiv.mulLeft₀ {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :

Left multiplication by a nonzero element in a GroupWithZero is a permutation of the underlying type.

Equations
Instances For
    @[simp]
    theorem Equiv.mulLeft₀_apply {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :
    (Equiv.mulLeft₀ a ha) = fun (x : G₀) => a * x
    @[simp]
    theorem Equiv.mulLeft₀_symm_apply {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :
    (Equiv.symm (Equiv.mulLeft₀ a ha)) = fun (x : G₀) => a⁻¹ * x
    theorem mulLeft_bijective₀ {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :
    Function.Bijective fun (x : G₀) => a * x
    def Equiv.mulRight₀ {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :

    Right multiplication by a nonzero element in a GroupWithZero is a permutation of the underlying type.

    Equations
    Instances For
      @[simp]
      theorem Equiv.mulRight₀_apply {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :
      (Equiv.mulRight₀ a ha) = fun (x : G₀) => x * a
      @[simp]
      theorem Equiv.mulRight₀_symm_apply {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :
      (Equiv.symm (Equiv.mulRight₀ a ha)) = fun (x : G₀) => x * a⁻¹
      theorem mulRight_bijective₀ {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :
      Function.Bijective fun (x : G₀) => x * a
      def Equiv.divRight₀ {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) :
      G₀ G₀

      Right division by a nonzero element in a GroupWithZero is a permutation of the underlying type.

      Equations
      • Equiv.divRight₀ a ha = { toFun := fun (x : G₀) => x / a, invFun := fun (x : G₀) => x * a, left_inv := , right_inv := }
      Instances For
        @[simp]
        theorem Equiv.divRight₀_symm_apply {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) (x✝ : G₀) :
        (Equiv.divRight₀ a ha).symm x✝ = x✝ * a
        @[simp]
        theorem Equiv.divRight₀_apply {G₀ : Type u_1} [GroupWithZero G₀] (a : G₀) (ha : a 0) (x✝ : G₀) :
        (Equiv.divRight₀ a ha) x✝ = x✝ / a