Algebra structures on the multiplicative opposite #
Main definitions #
MulOpposite.instAlgebra: the algebra onAᵐᵒᵖAlgHom.op/AlgHom.unop: simultaneously convert the domain and codomain of a morphism to the opposite algebra.AlgHom.opComm: swap which side of a morphism lies in the opposite algebra.AlgEquiv.op/AlgEquiv.unop: simultaneously convert the source and target of an isomorphism to the opposite algebra.AlgEquiv.opOp: any algebra is isomorphic to the opposite of its opposite.AlgEquiv.toOpposite: in a commutative algebra, the opposite algebra is isomorphic to the original algebra.AlgEquiv.opComm: swap which side of an isomorphism lies in the opposite algebra.
Equations
- MulOpposite.instAlgebra = { toSMul := MulOpposite.instSMul, algebraMap := (algebraMap R A).toOpposite ⋯, commutes' := ⋯, smul_def' := ⋯ }
An algebra is isomorphic to the opposite of its opposite.
Equations
- AlgEquiv.opOp R A = { toEquiv := (RingEquiv.opOp A).toEquiv, map_mul' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
An algebra homomorphism f : A →ₐ[R] B such that f x commutes with f y for all x, y defines
an algebra homomorphism from Aᵐᵒᵖ.
Equations
- f.fromOpposite hf = { toFun := ⇑f ∘ MulOpposite.unop, map_one' := ⋯, map_mul' := ⋯, map_zero' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
An algebra homomorphism f : A →ₐ[R] B such that f x commutes with f y for all x, y defines
an algebra homomorphism to Bᵐᵒᵖ.
Equations
- f.toOpposite hf = { toFun := MulOpposite.op ∘ ⇑f, map_one' := ⋯, map_mul' := ⋯, map_zero' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
An algebra hom A →ₐ[R] B can equivalently be viewed as an algebra hom Aᵐᵒᵖ →ₐ[R] Bᵐᵒᵖ.
This is the action of the (fully faithful) ᵐᵒᵖ-functor on morphisms.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The 'unopposite' of an algebra hom Aᵐᵒᵖ →ₐ[R] Bᵐᵒᵖ. Inverse to RingHom.op.
Equations
Instances For
Swap the ᵐᵒᵖ on an algebra hom to the opposite side.
Equations
Instances For
An algebra iso A ≃ₐ[R] B can equivalently be viewed as an algebra iso Aᵐᵒᵖ ≃ₐ[R] Bᵐᵒᵖ.
This is the action of the (fully faithful) ᵐᵒᵖ-functor on morphisms.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The 'unopposite' of an algebra iso Aᵐᵒᵖ ≃ₐ[R] Bᵐᵒᵖ. Inverse to AlgEquiv.op.
Equations
Instances For
Swap the ᵐᵒᵖ on an algebra isomorphism to the opposite side.
Equations
Instances For
The canonical algebra isomorphism from Aᵐᵒᵖ to Module.End A A induced by the right
multiplication.
Equations
- AlgEquiv.moduleEndSelf R = { toEquiv := (RingEquiv.moduleEndSelf A).toEquiv, map_mul' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
The canonical algebra isomorphism from A to Module.End Aᵐᵒᵖ A induced by the left
multiplication.
Equations
- AlgEquiv.moduleEndSelfOp R = { toEquiv := (RingEquiv.moduleEndSelfOp A).toEquiv, map_mul' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
A commutative algebra is isomorphic to its opposite.
Equations
- AlgEquiv.toOpposite R A = { toEquiv := (RingEquiv.toOpposite A).toEquiv, map_mul' := ⋯, map_add' := ⋯, commutes' := ⋯ }