Local rings #
Define local rings as commutative rings having a unique maximal ideal.
Main definitions #
- LocalRing: A predicate on commutative semirings, stating that for any pair of elements that adds up to- 1, one of them is a unit. This is shown to be equivalent to the condition that there exists a unique maximal ideal.
- LocalRing.maximalIdeal: The unique maximal ideal for a local rings. Its carrier set is the set of non units.
- IsLocalRingHom: A predicate on semiring homomorphisms, requiring that it maps nonunits to nonunits. For local rings, this means that the image of the unique maximal ideal is again contained in the unique maximal ideal.
- LocalRing.ResidueField: The quotient of a local ring by its maximal ideal.
A semiring is local if it is nontrivial and a or b is a unit whenever a + b = 1.
Note that LocalRing is a predicate.
- of_is_unit_or_is_unit_of_add_one :: (
- exists_pair_ne : ∃ (x : R) (y : R), x ≠ y
- in a local ring - R, if- a + b = 1, then either- ais a unit or- bis a unit. In another word, for every- a : R, either- ais a unit or- 1 - ais a unit.
- )
Instances
A semiring is local if it is nontrivial and the set of nonunits is closed under the addition.
A semiring is local if it has a unique maximal ideal.
The ideal of elements that are not units.
Equations
- LocalRing.maximalIdeal R = { carrier := nonunits R, add_mem' := ⋯, zero_mem' := ⋯, smul_mem' := ⋯ }
Instances For
Equations
- ⋯ = ⋯
A local ring homomorphism is a homomorphism f between local rings such that a in the domain
is a unit if f a is a unit for any a. See LocalRing.local_hom_TFAE for other equivalent
definitions.
- A local ring homomorphism - f : R ⟶ Swill send nonunits of- Rto nonunits of- S.
Instances
A local ring homomorphism f : R ⟶ S will send nonunits of R to nonunits of S.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
If f : R →+* S is a local ring hom, then R is a local ring if S is.
The image of the maximal ideal of the source is contained within the maximal ideal of the target.
A ring homomorphism between local rings is a local ring hom iff it reflects units, i.e. any preimage of a unit is still a unit. https://stacks.math.columbia.edu/tag/07BJ
If f : R →+* S is a surjective local ring hom, then the induced units map is surjective.
The residue field of a local ring is the quotient of the ring by its maximal ideal.
Equations
Instances For
Equations
- LocalRing.ResidueFieldCommRing R = let_fun this := inferInstance; this
Equations
- LocalRing.ResidueFieldInhabited R = let_fun this := inferInstance; this
Equations
The quotient map from a local ring to its residue field.
Equations
Instances For
Equations
Equations
- ⋯ = ⋯
A local ring homomorphism into a field can be descended onto the residue field.
Equations
Instances For
The map on residue fields induced by a local homomorphism between local rings
Equations
- LocalRing.ResidueField.map f = Ideal.Quotient.lift (LocalRing.maximalIdeal R) ((Ideal.Quotient.mk (LocalRing.maximalIdeal S)).comp f) ⋯
Instances For
Applying LocalRing.ResidueField.map to the identity ring homomorphism gives the identity
ring homomorphism.
The composite of two LocalRing.ResidueField.maps is the LocalRing.ResidueField.map of the
composite.
A ring isomorphism defines an isomorphism of residue fields.
Equations
- LocalRing.ResidueField.mapEquiv f = { toFun := ⇑(LocalRing.ResidueField.map ↑f), invFun := ⇑(LocalRing.ResidueField.map ↑f.symm), left_inv := ⋯, right_inv := ⋯, map_mul' := ⋯, map_add' := ⋯ }
Instances For
If G acts on R as a MulSemiringAction, then it also acts on LocalRing.ResidueField R.
Equations
- LocalRing.ResidueField.instMulSemiringAction G = MulSemiringAction.compHom (LocalRing.ResidueField R) (LocalRing.ResidueField.mapAut.comp (MulSemiringAction.toRingAut G R))