Isomorphisms of R
-algebras #
This file defines bundled isomorphisms of R
-algebras.
Main definitions #
AlgEquiv R A B
: the type ofR
-algebra isomorphisms betweenA
andB
.
Notations #
A ≃ₐ[R] B
:R
-algebra equivalence fromA
toB
.
- toFun : A → B
- invFun : B → A
- left_inv : Function.LeftInverse s.invFun s.toFun
- right_inv : Function.RightInverse s.invFun s.toFun
- map_mul' : ∀ (x y : A), Equiv.toFun s.toEquiv (x * y) = Equiv.toFun s.toEquiv x * Equiv.toFun s.toEquiv y
The proposition that the function preserves multiplication
- map_add' : ∀ (x y : A), Equiv.toFun s.toEquiv (x + y) = Equiv.toFun s.toEquiv x + Equiv.toFun s.toEquiv y
The proposition that the function preserves addition
- commutes' : ∀ (r : R), Equiv.toFun s.toEquiv (↑(algebraMap R A) r) = ↑(algebraMap R B) r
An equivalence of algebras commutes with the action of scalars.
An equivalence of algebras is an equivalence of rings commuting with the actions of scalars.
Instances For
An equivalence of algebras is an equivalence of rings commuting with the actions of scalars.
Instances For
- coe : F → A → B
- inv : F → B → A
- left_inv : ∀ (e : F), Function.LeftInverse (EquivLike.inv e) (EquivLike.coe e)
- right_inv : ∀ (e : F), Function.RightInverse (EquivLike.inv e) (EquivLike.coe e)
- coe_injective' : ∀ (e g : F), EquivLike.coe e = EquivLike.coe g → EquivLike.inv e = EquivLike.inv g → e = g
- commutes : ∀ (f : F) (r : R), ↑f (↑(algebraMap R A) r) = ↑(algebraMap R B) r
An equivalence of algebras commutes with the action of scalars.
AlgEquivClass F R A B
states that F
is a type of algebra structure preserving
equivalences. You should extend this class when you extend AlgEquiv
.
Instances
Turn an element of a type F
satisfying AlgEquivClass F R A B
into an actual AlgEquiv
.
This is declared as the default coercion from F
to A ≃ₐ[R] B
.
Instances For
Interpret an algebra equivalence as an algebra homomorphism.
This definition is included for symmetry with the other to*Hom
projections.
The simp
normal form is to use the coercion of the AlgHomClass.coeTC
instance.
Instances For
Algebra equivalences are reflexive.
Instances For
If A₁
is equivalent to A₁'
and A₂
is equivalent to A₂'
, then the type of maps
A₁ →ₐ[R] A₂
is equivalent to the type of maps A₁' →ₐ[R] A₂'
.
Instances For
If A₁
is equivalent to A₂
and A₁'
is equivalent to A₂'
, then the type of maps
A₁ ≃ₐ[R] A₁'
is equivalent to the type of maps A₂ ≃ ₐ[R] A₂'
.
This is the AlgEquiv
version of AlgEquiv.arrowCongr
.
Instances For
If an algebra morphism has an inverse, it is an algebra isomorphism.
Instances For
Promotes a bijective algebra homomorphism to an algebra equivalence.
Instances For
Upgrade a linear equivalence to an algebra equivalence, given that it distributes over multiplication and action of scalars.
Instances For
Promotes a linear ring_equiv to an AlgEquiv.
Instances For
An algebra isomorphism induces a group isomorphism between automorphism groups.
This is a more bundled version of AlgEquiv.equivCongr
.
Instances For
The tautological action by A₁ ≃ₐ[R] A₁
on A₁
.
This generalizes Function.End.applyMulAction
.
Each element of the group defines an algebra equivalence.
This is a stronger version of MulSemiringAction.toRingEquiv
and
DistribMulAction.toLinearEquiv
.