Ideal quotients #
This file defines ideal quotients as a special case of submodule quotients and proves some basic results about these quotients.
See Algebra.RingQuot
for quotients of non-commutative rings.
Main definitions #
Main results #
Ideal.quotientInfRingEquivPiQuotient
: the Chinese Remainder Theorem
The quotient R/I
of a ring R
by an ideal I
.
The ideal quotient of I
is defined to equal the quotient of I
as an R
-submodule of R
.
This definition is marked reducible
so that typeclass instances can be shared between
Ideal.Quotient I
and Submodule.Quotient I
.
On Ideal
s, Submodule.quotientRel
is a ring congruence.
Instances For
Two RingHom
s from the quotient by an ideal are equal if their
compositions with Ideal.Quotient.mk'
are equal.
See note [partially-applied ext lemmas].
If I
is an ideal of a commutative ring R
, if q : R → R/I
is the quotient map, and if
s ⊆ R
is a subset, then q⁻¹(q(s)) = ⋃ᵢ(i + s)
, the union running over all i ∈ I
.
The quotient by a maximal ideal is a group with zero. This is a def
rather than instance
,
since users will have computable inverses in some applications.
See note [reducible non-instances].
Instances For
The quotient by a maximal ideal is a field. This is a def
rather than instance
, since users
will have computable inverses (and qsmul
, rat_cast
) in some applications.
See note [reducible non-instances].
Instances For
The quotient of a ring by an ideal is a field iff the ideal is maximal.