Ideals in free modules over PIDs #
Main results #
Ideal.quotientEquivPiSpan
:S ⧸ I
, ifS
is finite free as a module over a PIDR
, can be written as a product of quotients ofR
by principal ideals.
noncomputable def
Ideal.quotientEquivPiSpan
{ι : Type u_1}
{R : Type u_2}
{S : Type u_3}
[CommRing R]
[CommRing S]
[Algebra R S]
[IsDomain R]
[IsPrincipalIdealRing R]
[IsDomain S]
[Finite ι]
(I : Ideal S)
(b : Basis ι R S)
(hI : I ≠ ⊥)
:
We can write the quotient of an ideal over a PID as a product of quotients by principal ideals.
Equations
- I.quotientEquivPiSpan b hI = (Submodule.restrictScalars R I).quotientEquivPiSpan b ⋯
Instances For
noncomputable def
Ideal.quotientEquivPiZMod
{ι : Type u_1}
{S : Type u_3}
[CommRing S]
[IsDomain S]
[Finite ι]
(I : Ideal S)
(b : Basis ι ℤ S)
(hI : I ≠ ⊥)
:
Ideal quotients over a free finite extension of ℤ
are isomorphic to a direct product of
ZMod
.
Equations
- I.quotientEquivPiZMod b hI = (Submodule.restrictScalars ℤ I).quotientEquivPiZMod b ⋯
Instances For
theorem
Ideal.finiteQuotientOfFreeOfNeBot
{S : Type u_3}
[CommRing S]
[IsDomain S]
[Module.Free ℤ S]
[Module.Finite ℤ S]
(I : Ideal S)
(hI : I ≠ ⊥)
:
A nonzero ideal over a free finite extension of ℤ
has a finite quotient.
It can't be an instance because of the side condition I ≠ ⊥
.
@[deprecated Ideal.finiteQuotientOfFreeOfNeBot (since := "2025-03-15")]
theorem
Ideal.fintypeQuotientOfFreeOfNeBot
{S : Type u_3}
[CommRing S]
[IsDomain S]
[Module.Free ℤ S]
[Module.Finite ℤ S]
(I : Ideal S)
(hI : I ≠ ⊥)
:
Alias of Ideal.finiteQuotientOfFreeOfNeBot
.
A nonzero ideal over a free finite extension of ℤ
has a finite quotient.
It can't be an instance because of the side condition I ≠ ⊥
.
noncomputable def
Ideal.quotientEquivDirectSum
{ι : Type u_1}
{R : Type u_2}
{S : Type u_3}
[CommRing R]
[CommRing S]
[Algebra R S]
[IsDomain R]
[IsPrincipalIdealRing R]
[IsDomain S]
[Finite ι]
(F : Type u_4)
[CommRing F]
[Algebra F R]
[Algebra F S]
[IsScalarTower F R S]
(b : Basis ι R S)
{I : Ideal S}
(hI : I ≠ ⊥)
:
Decompose S⧸I
as a direct sum of cyclic R
-modules
(quotients by the ideals generated by Smith coefficients of I
).
Equations
Instances For
theorem
Ideal.finrank_quotient_eq_sum
{R : Type u_2}
{S : Type u_3}
[CommRing R]
[CommRing S]
[Algebra R S]
[IsDomain R]
[IsPrincipalIdealRing R]
[IsDomain S]
(F : Type u_4)
[CommRing F]
[Algebra F R]
[Algebra F S]
[IsScalarTower F R S]
{I : Ideal S}
(hI : I ≠ ⊥)
{ι : Type u_5}
[Fintype ι]
(b : Basis ι R S)
[Nontrivial F]
[∀ (i : ι), Module.Free F (R ⧸ span {smithCoeffs b I hI i})]
[∀ (i : ι), Module.Finite F (R ⧸ span {smithCoeffs b I hI i})]
: