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 semirings.
Main definitions #
Equations
- Ideal.Quotient.instUniqueQuotientTop = { default := 0, uniq := ⋯ }
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].
Equations
- Ideal.Quotient.groupWithZero I = GroupWithZero.mk ⋯ zpowRec ⋯ ⋯ ⋯ ⋯ ⋯
Instances For
The quotient by a two-sided ideal that is maximal as a left ideal is a division ring.
This is a def
rather than instance
, since users
will have computable inverses (and qsmul
, ratCast
) in some applications.
See note [reducible non-instances].
Equations
- Ideal.Quotient.divisionRing I = DivisionRing.mk ⋯ GroupWithZero.zpow ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ (fun (x : ℚ≥0) => HMul.hMul ↑x) ⋯ ⋯ (fun (x : ℚ) => HMul.hMul ↑x) ⋯
Instances For
The quotient of a commutative ring by a maximal ideal is a field.
This is a def
rather than instance
, since users
will have computable inverses (and qsmul
, ratCast
) in some applications.
See note [reducible non-instances].
Equations
- Ideal.Quotient.field I = Field.mk ⋯ DivisionRing.zpow ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ DivisionRing.nnqsmul ⋯ ⋯ DivisionRing.qsmul ⋯
Instances For
A ring is made up of a disjoint union of cosets of an ideal.