Ideals in a matrix ring #
This file defines left (resp. two-sided) ideals in a matrix semiring (resp. ring) over left (resp. two-sided) ideals in the base semiring (resp. ring). We also characterize Jacobson radicals of ideals in such rings.
Main results #
TwoSidedIdeal.equivMatricesOver
andTwoSidedIdeal.orderIsoMatricesOver
establish an order isomorphism between two-sided ideals in $R$ and those in $Mₙ(R)$.TwoSidedIdeal.jacobson_matricesOver
shows that $J(Mₙ(I)) = Mₙ(J(I))$ for any two-sided ideal $I ≤ R$.
Left ideals in a matrix semiring #
The left ideal of matrices with entries in I ≤ R
.
Equations
- Ideal.matricesOver n I = { carrier := {M : Matrix n n R | ∀ (i j : n), M i j ∈ I}, add_mem' := ⋯, zero_mem' := ⋯, smul_mem' := ⋯ }
Instances For
Jacobson radicals of left ideals in a matrix ring #
A standard basis matrix is in $J(Mₙ(I))$ as long as its one possibly non-zero entry is in $J(I)$.
For any left ideal $I ≤ R$, we have $Mₙ(J(I)) ≤ J(Mₙ(I))$.
Two-sided ideals in a matrix ring #
The two-sided ideal of matrices with entries in I ≤ R
.
Equations
- TwoSidedIdeal.matricesOver n I = TwoSidedIdeal.mk' {M : Matrix n n R | ∀ (i j : n), M i j ∈ I} ⋯ ⋯ ⋯ ⋯ ⋯
Instances For
Two-sided ideals in $R$ correspond bijectively to those in $Mₙ(R)$. Given an ideal $I ≤ R$, we send it to $Mₙ(I)$. Given an ideal $J ≤ Mₙ(R)$, we send it to $\{Nᵢⱼ ∣ ∃ N ∈ J\}$.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Two-sided ideals in $R$ are order-isomorphic with those in $Mₙ(R)$.
See also equivMatricesOver
.
Equations
- TwoSidedIdeal.orderIsoMatricesOver i j = { toEquiv := TwoSidedIdeal.equivMatricesOver i j, map_rel_iff' := ⋯ }
Instances For
Jacobson radicals of two-sided ideals in a matrix ring #
For any two-sided ideal $I ≤ R$, we have $J(Mₙ(I)) = Mₙ(J(I))$.