Isotypic modules and isotypic components #
Main definitions #
IsIsotypicOfType R M S
means that all simple submodules of theR
-moduleM
are isomorphic toS
. Such a moduleM
is isomorphic to a finsupp overS
, seeIsIsotypicOfType.linearEquiv_finsupp
.IsIsotypic R M
means that all simple submodules of theR
-moduleM
are isomorphic to each other.isotypicComponent R M S
is the sum of all submodules ofM
isomorphic toS
.isotypicComponents R M
is the set of all nontrivial isotypic components ofM
(whereS
is taken to be simple submodules).Submodule.IsFullyInvariant N
means that the submoduleN
of anR
-moduleM
is mapped into itself by all endomorphisms ofM
. ThefullyInvariantSubmodule
s ofM
form a complete lattice, which is atomic ifM
is semisimple, in which case the atoms are the isotypic components ofM
. A fully invariant submodule of a semiring as a module over itself is simply a two-sided ideal, seeisFullyInvariant_iff_isTwoSided
.iSupIndep.ringEquiv
,iSupIndep.algEquiv
: ifM
is the direct sum of fully invariant submodulesNᵢ
, thenEnd R M
is isomorphic toΠᵢ End R Nᵢ
. This can be applied to the isotypic components of a semisimple moduleM
, yieldingIsSemisimpleModule.endAlgEquiv
.
Keywords #
isotypic component, fully invariant submodule
An R
-module M
is isotypic of type S
if all simple submodules of M
are isomorphic
to S
. If M
is semisimple, it is equivalent to requiring that all simple quotients of M
are
isomorphic to S
.
Equations
- IsIsotypicOfType R M S = ∀ (m : Submodule R M) [IsSimpleModule R ↥m], Nonempty (↥m ≃ₗ[R] S)
Instances For
An R
-module M
is isotypic if all its simple submodules are isomorphic.
Equations
- IsIsotypic R M = ∀ (m : Submodule R M) [IsSimpleModule R ↥m], IsIsotypicOfType R M ↥m
Instances For
If S
is a simple R
-module, the S
-isotypic component in an R
-module M
is the sum of
all submodules of M
isomorphic to S
.
Instances For
The set of all (nontrivial) isotypic components of a module.
Equations
- isotypicComponents R M = {m : Submodule R M | ∃ (S : Submodule R M), IsSimpleModule R ↥S ∧ m = isotypicComponent R M ↥S}
Instances For
If a simple module is contained in a sum of semisimple modules, it must be isomorphic to a submodule of one of the summands.
A submodule N
an R
-module M
is fully invariant if N
is mapped into itself by all
R
-linear endomorphisms of M
.
If M
is semisimple, this is equivalent to N
being a sum of isotypic components of M
:
see isFullyInvariant_iff_sSup_isotypicComponents
.
Equations
- N.IsFullyInvariant = ∀ (f : Module.End R M), N ≤ Submodule.comap f N
Instances For
The fully invariant submodules of a module form a complete sublattice in the lattice of submodules.
Equations
- fullyInvariantSubmodule R M = CompleteSublattice.mk' {N : Submodule R M | N.IsFullyInvariant} ⋯ ⋯
Instances For
If an R
-module M
is the direct sum of fully invariant submodules Nᵢ
,
then End R M
is isomorphic to Πᵢ End R Nᵢ
as a ring.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If an R
-module M
is the direct sum of fully invariant submodules Nᵢ
,
then End R M
is isomorphic to Πᵢ End R Nᵢ
as an algebra.
Equations
Instances For
The Galois coinsertion from sets of isotypic components to fully invariant submodules.
Equations
Instances For
Sets of isotypic components in a semisimple module are in order-preserving 1-1 correspondence with fully invariant submodules. Consequently, the fully invariant submodules form a complete atomic Boolean algebra.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The endomorphism algebra of a semisimple module is the direct product of the endomorphism algebras of its isotypic components.
Equations
- IsSemisimpleModule.endAlgEquiv R₀ R M = iSupIndep.algEquiv R₀ ⋯ ⋯ ⋯
Instances For
The endomorphism ring of a semisimple module is the direct product of the endomorphism rings of its isotypic components.