Documentation

Mathlib.RingTheory.LocalRing.RingHom.Basic

Local rings homomorphisms #

We prove basic properties of local rings homomorphisms.

Equations
  • =
@[simp]
theorem isUnit_map_iff {R : Type u_1} {S : Type u_2} [Semiring R] [Semiring S] (f : R →+* S) [IsLocalRingHom f] (a : R) :
IsUnit (f a) IsUnit a
@[simp]
theorem map_mem_nonunits_iff {R : Type u_1} {S : Type u_2} [Semiring R] [Semiring S] (f : R →+* S) [IsLocalRingHom f] (a : R) :
instance isLocalRingHom_comp {R : Type u_1} {S : Type u_2} {T : Type u_3} [Semiring R] [Semiring S] [Semiring T] (g : S →+* T) (f : R →+* S) [IsLocalRingHom g] [IsLocalRingHom f] :
IsLocalRingHom (g.comp f)
Equations
  • =
instance isLocalRingHom_equiv {R : Type u_1} {S : Type u_2} [Semiring R] [Semiring S] (f : R ≃+* S) :
Equations
  • =
@[simp]
theorem isUnit_of_map_unit {R : Type u_1} {S : Type u_2} [Semiring R] [Semiring S] (f : R →+* S) [IsLocalRingHom f] (a : R) (h : IsUnit (f a)) :
theorem of_irreducible_map {R : Type u_1} {S : Type u_2} [Semiring R] [Semiring S] (f : R →+* S) [h : IsLocalRingHom f] {x : R} (hfx : Irreducible (f x)) :
theorem isLocalRingHom_of_comp {R : Type u_1} {S : Type u_2} {T : Type u_3} [Semiring R] [Semiring S] [Semiring T] (f : R →+* S) (g : S →+* T) [IsLocalRingHom (g.comp f)] :
theorem RingHom.domain_localRing {R : Type u_4} {S : Type u_5} [CommSemiring R] [CommSemiring S] [H : LocalRing S] (f : R →+* S) [IsLocalRingHom f] :

If f : R →+* S is a local ring hom, then R is a local ring if S is.

theorem map_nonunit {R : Type u_1} {S : Type u_2} [CommSemiring R] [LocalRing R] [CommSemiring S] [LocalRing S] (f : R →+* S) [IsLocalRingHom f] (a : R) (h : a LocalRing.maximalIdeal R) :

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.

@[instance 100]

Every ring hom f : K →+* R from a division ring K to a nontrivial ring R is a local ring hom.

Equations
  • =
theorem RingEquiv.localRing {A : Type u_4} {B : Type u_5} [CommSemiring A] [LocalRing A] [CommSemiring B] (e : A ≃+* B) :