Internally-graded rings and algebras #
This file defines the typeclass graded_algebra 𝒜
, for working with an algebra A
that is
internally graded by a collection of submodules 𝒜 : ι → submodule R A
.
See the docstring of that typeclass for more information.
Main definitions #
graded_ring 𝒜
: the typeclass, which is a combination ofset_like.graded_monoid
, anddirect_sum.decomposition 𝒜
.graded_algebra 𝒜
: A convenience alias forgraded_ring
when𝒜
is a family of submodules.direct_sum.decompose_ring_equiv 𝒜 : A ≃ₐ[R] ⨁ i, 𝒜 i
, a more bundled version ofdirect_sum.decompose 𝒜
.direct_sum.decompose_alg_equiv 𝒜 : A ≃ₐ[R] ⨁ i, 𝒜 i
, a more bundled version ofdirect_sum.decompose 𝒜
.graded_algebra.proj 𝒜 i
is the linear map fromA
to its degreei : ι
component, such thatproj 𝒜 i x = decompose 𝒜 x i
.
Implementation notes #
For now, we do not have internally-graded semirings and internally-graded rings; these can be
represented with 𝒜 : ι → submodule ℕ A
and 𝒜 : ι → submodule ℤ A
respectively, since all
semiring
s are ℕ-algebras via algebra_nat
, and all ring
s are ℤ
-algebras via algebra_int
.
Tags #
graded algebra, graded ring, graded semiring, decomposition
- to_graded_monoid : set_like.graded_monoid 𝒜
- to_decomposition : direct_sum.decomposition 𝒜
An internally-graded R
-algebra A
is one that can be decomposed into a collection
of submodule R A
s indexed by ι
such that the canonical map A → ⨁ i, 𝒜 i
is bijective and
respects multiplication, i.e. the product of an element of degree i
and an element of degree j
is an element of degree i + j
.
Note that the fact that A
is internally-graded, graded_algebra 𝒜
, implies an externally-graded
algebra structure direct_sum.galgebra R (λ i, ↥(𝒜 i))
, which in turn makes available an
algebra R (⨁ i, 𝒜 i)
instance.
Instances of this typeclass
Instances of other typeclasses for graded_ring
- graded_ring.has_sizeof_inst
If A
is graded by ι
with degree i
component 𝒜 i
, then it is isomorphic as
a ring to a direct sum of components.
The projection maps of a graded ring
Equations
A special case of graded_ring
with σ = submodule R A
. This is useful both because it
can avoid typeclass search, and because it provides a more concise name.
Equations
A helper to construct a graded_algebra
when the set_like.graded_monoid
structure is already
available. This makes the left_inv
condition easier to prove, and phrases the right_inv
condition in a way that allows custom @[ext]
lemmas to apply.
See note [reducible non-instances].
Equations
- graded_algebra.of_alg_hom 𝒜 decompose right_inv left_inv = graded_ring.mk
If A
is graded by ι
with degree i
component 𝒜 i
, then it is isomorphic as
an algebra to a direct sum of components.
The projection maps of graded algebra
Equations
- graded_algebra.proj 𝒜 i = (𝒜 i).subtype.comp ((dfinsupp.lapply i).comp (direct_sum.decompose_alg_equiv 𝒜).to_alg_hom.to_linear_map)
If A
is graded by a canonically ordered add monoid, then the projection map x ↦ x₀
is a ring
homomorphism.