Skip to content

Commit

Permalink
fixing error after adding change
Browse files Browse the repository at this point in the history
  • Loading branch information
maddycrim committed Oct 30, 2024
1 parent 037ace6 commit c6c8da1
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -128,7 +128,7 @@ noncomputable def nilradmaxlocalizationIsSelf [h : (nilradical R).IsMaximal] (h'
[IsLocalization M S] : R ≃ₐ[R] S := by
have (m) (hm : m ∈ M) : IsUnit m := by
haveI := LocalRing.of_nilradical_isMaximal (h := h)
apply (LocalRing.not_mem_maximalIdeal m).mp
apply LocalRing.not_mem_maximalIdeal.mp
rw [← LocalRing.eq_maximalIdeal h]
rintro ⟨k, hk⟩
rw [← hk] at h'
Expand Down

0 comments on commit c6c8da1

Please sign in to comment.