File tree Expand file tree Collapse file tree 2 files changed +4
-10
lines changed Expand file tree Collapse file tree 2 files changed +4
-10
lines changed Original file line number Diff line number Diff line change @@ -187,13 +187,8 @@ end FiniteDimensional
187187
188188end ResidueField
189189
190- theorem isLocalHom_residue : IsLocalHom (IsLocalRing.residue R) := by
191- constructor
192- intro a ha
193- by_contra h
194- rw [residue_def, Ideal.Quotient.eq_zero_iff_mem.mpr ((IsLocalRing.mem_maximalIdeal _).mpr h)]
195- at ha
196- exact ha.ne_zero rfl
190+ @[deprecated (since := "2025-10-06")]
191+ alias isLocalHom_residue := instIsLocalHomResidueFieldRingHomResidue
197192
198193end
199194
Original file line number Diff line number Diff line change @@ -642,9 +642,8 @@ theorem ker_unitGroupToResidueFieldUnits :
642642
643643theorem surjective_unitGroupToResidueFieldUnits :
644644 Function.Surjective A.unitGroupToResidueFieldUnits :=
645- (IsLocalRing.surjective_units_map_of_local_ringHom _ Ideal.Quotient.mk_surjective
646- IsLocalRing.isLocalHom_residue).comp
647- (MulEquiv.surjective _)
645+ IsLocalRing.surjective_units_map_of_local_ringHom _ Ideal.Quotient.mk_surjective
646+ (inferInstanceAs (IsLocalHom (IsLocalRing.residue A))) |>.comp (MulEquiv.surjective _)
648647
649648/-- The quotient of the unit group of `A` by the principal unit group of `A` agrees with
650649the units of the residue field of `A`. -/
You can’t perform that action at this time.
0 commit comments