More operations on modules and ideals related to quotients #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
The induced map from the quotient by the kernel to the codomain.
This is an isomorphism if f
has a right inverse (quotient_ker_equiv_of_right_inverse
) /
is surjective (quotient_ker_equiv_of_surjective
).
Equations
- f.ker_lift = ideal.quotient.lift (ring_hom.ker f) f _
The first isomorphism theorem for commutative rings, computable version.
Equations
- ring_hom.quotient_ker_equiv_of_right_inverse hf = {to_fun := ⇑(f.ker_lift), inv_fun := ⇑(ideal.quotient.mk (ring_hom.ker f)) ∘ g, left_inv := _, right_inv := hf, map_mul' := _, map_add' := _}
The first isomorphism theorem for commutative rings.
See also ideal.mem_quotient_iff_mem
in case I ≤ J
.
See also ideal.mem_quotient_iff_mem_sup
if the assumption I ≤ J
is not available.
The R₁
-algebra structure on A/I
for an R₁
-algebra A
Equations
- ideal.quotient.algebra R₁ = {to_has_smul := {smul := has_smul.smul (submodule.quotient.has_smul' I)}, to_ring_hom := {to_fun := λ (x : R₁), ⇑(ideal.quotient.mk I) (⇑(algebra_map R₁ A) x), map_one' := _, map_mul' := _, map_zero' := _, map_add' := _}, commutes' := _, smul_def' := _}
The canonical morphism A →ₐ[R₁] A ⧸ I
as morphism of R₁
-algebras, for I
an ideal of
A
, where A
is an R₁
-algebra.
Equations
- ideal.quotient.mkₐ R₁ I = {to_fun := λ (a : A), submodule.quotient.mk a, map_one' := _, map_mul' := _, map_zero' := _, map_add' := _, commutes' := _}
The canonical morphism A →ₐ[R₁] I.quotient
is surjective.
The kernel of A →ₐ[R₁] I.quotient
is I
.
The induced algebras morphism from the quotient by the kernel to the codomain.
This is an isomorphism if f
has a right inverse (quotient_ker_alg_equiv_of_right_inverse
) /
is surjective (quotient_ker_alg_equiv_of_surjective
).
Equations
The first isomorphism theorem for algebras, computable version.
Equations
- ideal.quotient_ker_alg_equiv_of_right_inverse hf = {to_fun := (ring_hom.quotient_ker_equiv_of_right_inverse _).to_fun, inv_fun := (ring_hom.quotient_ker_equiv_of_right_inverse _).inv_fun, left_inv := _, right_inv := _, map_mul' := _, map_add' := _, commutes' := _}
The first isomorphism theorem for algebras.
The ring hom R/I →+* S/J
induced by a ring hom f : R →+* S
with I ≤ f⁻¹(J)
Equations
- J.quotient_map f hIJ = ideal.quotient.lift I ((ideal.quotient.mk J).comp f) _
H
and h
are kept as separate hypothesis since H is used in constructing the quotient map.
If we take J = I.comap f
then quotient_map
is injective automatically.
Commutativity of a square is preserved when taking quotients by an ideal.
The algebra hom A/I →+* B/J
induced by an algebra hom f : A →ₐ[R₁] B
with I ≤ f⁻¹(J)
.
The algebra equiv A/I ≃ₐ[R] B/J
induced by an algebra equiv f : A ≃ₐ[R] B
,
whereJ = f(I)
.
Equations
- ideal.quotient_algebra = (I.quotient_map (algebra_map R A) ideal.quotient_algebra._proof_1).to_algebra
Quotienting by equal ideals gives equivalent algebras.
Equations
The obvious ring hom R/I → R/(I ⊔ J)
Equations
- double_quot.quot_left_to_quot_sup I J = ideal.quotient.factor I (I ⊔ J) _
The kernel of quot_left_to_quot_sup
The ring homomorphism (R/I)/J' -> R/(I ⊔ J)
induced by quot_left_to_quot_sup
where J'
is the image of J
in R/I
Equations
The composite of the maps R → (R/I)
and (R/I) → (R/I)/J'
Equations
- double_quot.quot_quot_mk I J = (ideal.quotient.mk (ideal.map (ideal.quotient.mk I) J)).comp (ideal.quotient.mk I)
The kernel of quot_quot_mk
The ring homomorphism R/(I ⊔ J) → (R/I)/J'
induced by quot_quot_mk
Equations
- double_quot.lift_sup_quot_quot_mk I J = ideal.quotient.lift (I ⊔ J) (double_quot.quot_quot_mk I J) _
quot_quot_to_quot_add
and lift_sup_double_qot_mk
are inverse isomorphisms. In the case where
I ≤ J
, this is the Third Isomorphism Theorem (see quot_quot_equiv_quot_of_le
)
Equations
The obvious isomorphism (R/I)/J' → (R/J)/I'
Equations
The Third Isomorphism theorem for rings. See quot_quot_equiv_quot_sup
for a version
that does not assume an inclusion of ideals.
Equations
The natural algebra homomorphism A / I → A / (I ⊔ J)
.
The algebra homomorphism (A / I) / J' -> A / (I ⊔ J) induced by
quot_left_to_quot_sup, where
J'is the projection of
Jin
A / I`.
The composition of the algebra homomorphisms A → (A / I)
and (A / I) → (A / I) / J'
,
where J'
is the projection J
in A / I
.
The injective algebra homomorphism A / (I ⊔ J) → (A / I) / J'
induced by quot_quot_mk
,
where J'
is the projection J
in A / I
.
quot_quot_to_quot_add
and lift_sup_quot_quot_mk
are inverse isomorphisms. In the case where
I ≤ J
, this is the Third Isomorphism Theorem (see quot_quot_equiv_quot_of_le
).
Equations
The natural algebra isomorphism (A / I) / J' → (A / J) / I'
,
where J'
(resp. I'
) is the projection of J
in A / I
(resp. I
in A / J
).
Equations
The third isomoprhism theorem for rings. See quot_quot_equiv_quot_sup
for version
that does not assume an inclusion of ideals.