Documentation

Mathlib.Algebra.GroupWithZero.Semiconj

Lemmas about semiconjugate elements in a GroupWithZero. #

@[simp]
theorem SemiconjBy.zero_right {G₀ : Type u_3} [MulZeroClass G₀] (a : G₀) :
@[simp]
theorem SemiconjBy.zero_left {G₀ : Type u_3} [MulZeroClass G₀] (x : G₀) (y : G₀) :
@[simp]
theorem SemiconjBy.inv_symm_left_iff₀ {G₀ : Type u_3} [GroupWithZero G₀] {a : G₀} {x : G₀} {y : G₀} :
theorem SemiconjBy.inv_symm_left₀ {G₀ : Type u_3} [GroupWithZero G₀] {a : G₀} {x : G₀} {y : G₀} (h : SemiconjBy a x y) :
theorem SemiconjBy.inv_right₀ {G₀ : Type u_3} [GroupWithZero G₀] {a : G₀} {x : G₀} {y : G₀} (h : SemiconjBy a x y) :
@[simp]
theorem SemiconjBy.inv_right_iff₀ {G₀ : Type u_3} [GroupWithZero G₀] {a : G₀} {x : G₀} {y : G₀} :
theorem SemiconjBy.div_right {G₀ : Type u_3} [GroupWithZero G₀] {a : G₀} {x : G₀} {y : G₀} {x' : G₀} {y' : G₀} (h : SemiconjBy a x y) (h' : SemiconjBy a x' y') :
SemiconjBy a (x / x') (y / y')