Skip to content

Commit

Permalink
feat(ring_theory/ideal/local_ring): add ​local_ring.residue_field.map…
Browse files Browse the repository at this point in the history
…_id & local_ring.residue_field.map_comp (#16916)

Applying `map` to the identity ring homomorphism gives the identity ring homomorphism. 

The composite of two `map`s is the `map` of the composite.

I need these for my study of the inertia group



Co-authored-by: mkaratarakis <40603357+mkaratarakis@users.noreply.github.com>
  • Loading branch information
mkaratarakis and mkaratarakis committed Oct 11, 2022
1 parent 2f93d81 commit bbcc67f
Showing 1 changed file with 13 additions and 1 deletion.
14 changes: 13 additions & 1 deletion src/ring_theory/ideal/local_ring.lean
Expand Up @@ -328,7 +328,7 @@ begin
end

section
variables (R) [comm_ring R] [local_ring R] [comm_ring S] [local_ring S]
variables (R) [comm_ring R] [local_ring R] [comm_ring S] [local_ring S] [comm_ring T] [local_ring T]

/-- The residue field of a local ring is the quotient of the ring by its maximal ideal. -/
def residue_field := R ⧸ maximal_ideal R
Expand Down Expand Up @@ -359,6 +359,18 @@ begin
exact map_nonunit f a ha
end

/-- Applying `residue_field.map` to the identity ring homomorphism gives the identity
ring homomorphism. -/
lemma map_id :
local_ring.residue_field.map (ring_hom.id R) = ring_hom.id (local_ring.residue_field R) :=
ideal.quotient.ring_hom_ext $ ring_hom.ext $ λx, rfl

/-- The composite of two `residue_field.map`s is the `residue_field.map` of the composite. -/
lemma map_comp (f : T →+* R) (g : R →+* S) [is_local_ring_hom f] [is_local_ring_hom g] :
local_ring.residue_field.map (g.comp f) =
(local_ring.residue_field.map g).comp (local_ring.residue_field.map f) :=
ideal.quotient.ring_hom_ext $ ring_hom.ext $ λx, rfl

end residue_field

lemma ker_eq_maximal_ideal [field K] (φ : R →+* K) (hφ : function.surjective φ) :
Expand Down

0 comments on commit bbcc67f

Please sign in to comment.