Multiplicative and additive equivalence acting on units. #
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Left addition of an additive unit is a permutation of the underlying type.
Left multiplication by a unit of a monoid is a permutation of the underlying type.
Right addition of an additive unit is a permutation of the underlying type.
Right multiplication by a unit of a monoid is a permutation of the underlying type.
Left addition in an AddGroup
is a permutation of the underlying type.
Equations
- Equiv.addLeft a = AddUnits.addLeft (↑toAddUnits a)
Left multiplication in a Group
is a permutation of the underlying type.
Equations
- Equiv.mulLeft a = Units.mulLeft (↑toUnits a)
Extra simp lemma that dsimp
can use. simp
will never use this.
Extra simp lemma that dsimp
can use. simp
will never use this.
Right addition in an AddGroup
is a permutation of the underlying type.
Equations
- Equiv.addRight a = AddUnits.addRight (↑toAddUnits a)
Right multiplication in a Group
is a permutation of the underlying type.
Equations
- Equiv.mulRight a = Units.mulRight (↑toUnits a)
Extra simp lemma that dsimp
can use. simp
will never use this.
Extra simp lemma that dsimp
can use. simp
will never use this.
A version of Equiv.addLeft a (-b)
that is defeq to a - b
.
A version of Equiv.mulLeft a b⁻¹⁻¹
that is defeq to a / b
.
A version of Equiv.addRight (-a) b
that is defeq to b - a
.
A version of Equiv.mulRight a⁻¹ b⁻¹ b
that is defeq to b / a
.
In a DivisionCommMonoid
, Equiv.inv
is a MulEquiv
. There is a variant of this
MulEquiv.inv' G : G ≃* Gᵐᵒᵖ≃* Gᵐᵒᵖ
for the non-commutative case.
Equations
- One or more equations did not get rendered due to their size.