Unitization of a non-unital algebra #
Given a non-unital R
-algebra A
(given via the type classes
[NonUnitalRing A] [Module R A] [SMulCommClass R A A] [IsScalarTower R A A]
) we construct
the minimal unital R
-algebra containing A
as an ideal. This object algebra.unitization R A
is
a type synonym for R × A
on which we place a different multiplicative structure, namely,
(r₁, a₁) * (r₂, a₂) = (r₁ * r₂, r₁ • a₂ + r₂ • a₁ + a₁ * a₂)
where the multiplicative identity
is (1, 0)
.
Note, when A
is a unital R
-algebra, then Unitization R A
constructs a new multiplicative
identity different from the old one, and so in general Unitization R A
and A
will not be
isomorphic even in the unital case. This approach actually has nice functorial properties.
There is a natural coercion from A
to Unitization R A
given by fun a ↦ (0, a)
, the image
of which is a proper ideal (TODO), and when R
is a field this ideal is maximal. Moreover,
this ideal is always an essential ideal (it has nontrivial intersection with every other nontrivial
ideal).
Every non-unital algebra homomorphism from A
into a unital R
-algebra B
has a unique
extension to a (unital) algebra homomorphism from Unitization R A
to B
.
Main definitions #
Unitization R A
: the unitization of a non-unitalR
-algebraA
.Unitization.algebra
: the unitization ofA
as a (unital)R
-algebra.Unitization.coeNonUnitalAlgHom
: coercion as a non-unital algebra homomorphism.NonUnitalAlgHom.toAlgHom φ
: the extension of a non-unital algebra homomorphismφ : A → B
into a unitalR
-algebraB
to an algebra homomorphismUnitization R A →ₐ[R] B
.Unitization.lift
: the universal property of the unitization, the extensionNonUnitalAlgHom.toAlgHom
actually implements an equivalence(A →ₙₐ[R] B) ≃ (Unitization R A ≃ₐ[R] B)
Main results #
AlgHom.ext'
: an extensionality lemma for algebra homomorphisms whose domain isUnitization R A
; it suffices that they agree onA
.
TODO #
- prove the unitization operation is a functor between the appropriate categories
- prove the image of the coercion is an essential ideal, maximal if scalars are a field.
The minimal unitization of a non-unital R
-algebra A
. This is just a type synonym for
R × A
.
Instances For
The canonical inclusion R → Unitization R A
.
Instances For
The canonical inclusion A → Unitization R A
.
Instances For
The canonical projection Unitization R A → R
.
Instances For
The canonical projection Unitization R A → A
.
Instances For
The identity map between Unitization R A
and R × A
as an AddEquiv
.
Instances For
To show a property hold on all Unitization R A
it suffices to show it holds
on terms of the form inl r + a
.
This can be used as induction x using Unitization.ind
.
This cannot be marked @[ext]
as it ends up being used instead of LinearMap.prod_ext
when
working with R × A
.
The canonical R
-linear inclusion A → Unitization R A
.
Instances For
The canonical R
-linear projection Unitization R A → A
.
Instances For
Multiplicative structure #
The canonical inclusion of rings R →+* Unitization R A
.
Instances For
Star structure #
Algebra structure #
The canonical R
-algebra projection Unitization R A → R
.
Instances For
The coercion from a non-unital R
-algebra A
to its unitization Unitization R A
realized as a non-unital algebra homomorphism.
Instances For
The coercion from a non-unital R
-algebra A
to its unitization unitization R A
realized as a non-unital star algebra homomorphism.
Instances For
See note [partially-applied ext lemmas]
A non-unital algebra homomorphism from A
into a unital R
-algebra C
lifts to a unital
algebra homomorphism from the unitization into C
. This is extended to an Equiv
in
Unitization.lift
and that should be used instead. This declaration only exists for performance
reasons.
Instances For
Non-unital algebra homomorphisms from A
into a unital R
-algebra C
lift uniquely to
Unitization R A →ₐ[R] C
. This is the universal property of the unitization.
Instances For
See note [partially-applied ext lemmas]
Non-unital star algebra homomorphisms from A
into a unital star R
-algebra C
lift uniquely
to Unitization R A →⋆ₐ[R] C
. This is the universal property of the unitization.