Towers of algebras
We set up the basic theory of algebra towers.
An algebra tower A/S/R is expressed by having instances of algebra A S
,
algebra R S
, algebra R A
and is_scalar_tower R S A
, the later asserting the
compatibility condition (r • s) • a = r • (s • a)
.
In field_theory/tower.lean
we use this to prove the tower law for finite extensions,
that if R
and S
are both fields, then [A:R] = [A:S] [S:A]
.
In this file we prepare the main lemma:
if {bi | i ∈ I}
is an R
-basis of S
and {cj | j ∈ J}
is a S
-basis
of A
, then {bi cj | i ∈ I, j ∈ J}
is an R
-basis of A
. This statement does not require the
base rings to be a field, so we also generalize the lemma to rings in this file.
In a tower, the canonical map from the middle element to the top element is an algebra homomorphism over the bottom element.
R ⟶ S induces S-Alg ⥤ R-Alg
If A/S/R is a tower of algebras then the res
triction of a S-subalgebra of A is an R-subalgebra of A.
Equations
- subalgebra.res R U = {carrier := U.carrier, one_mem' := _, mul_mem' := _, zero_mem' := _, add_mem' := _, algebra_map_mem' := _}
Produces a map from subalgebra.under
.
Restricting the scalars of submodules in an algebra tower.
Artin--Tate lemma: if A ⊆ B ⊆ C is a chain of subrings of commutative rings, and A is noetherian, and C is algebra-finite over A, and C is module-finite over B, then B is algebra-finite over A.
References: Atiyah--Macdonald Proposition 7.8; Stacks 00IS; Altman--Kleiman 16.17.