Skip to content

Commit e99565a

Browse files
committed
chore(RingTheory/Spectrum/Prime/Module): golf stableUnderSpecialization_support using mem_support_mono (#30148)
Golf [Module.stableUnderSpecialization_support](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Spectrum/Prime/Module.html#Module.stableUnderSpecialization_support) using [Module.mem_support_mono](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Support.html#Module.mem_support_mono).
1 parent 66464ac commit e99565a

File tree

1 file changed

+2
-6
lines changed

1 file changed

+2
-6
lines changed

Mathlib/RingTheory/Spectrum/Prime/Module.lean

Lines changed: 2 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -36,12 +36,8 @@ lemma LocalizedModule.subsingleton_iff_disjoint {f : R} :
3636
rw [subsingleton_iff_support_subset, PrimeSpectrum.basicOpen_eq_zeroLocus_compl,
3737
disjoint_compl_left_iff, Set.le_iff_subset]
3838

39-
lemma Module.stableUnderSpecialization_support :
40-
StableUnderSpecialization (Module.support R M) := by
41-
intro x y e H
42-
rw [mem_support_iff_exists_annihilator] at H ⊢
43-
obtain ⟨m, hm⟩ := H
44-
exact ⟨m, hm.trans ((PrimeSpectrum.le_iff_specializes _ _).mpr e)⟩
39+
lemma Module.stableUnderSpecialization_support : StableUnderSpecialization (Module.support R M) :=
40+
fun x y e ↦ mem_support_mono <| (PrimeSpectrum.le_iff_specializes x y).mpr e
4541

4642
lemma Module.isClosed_support [Module.Finite R M] :
4743
IsClosed (Module.support R M) := by

0 commit comments

Comments
 (0)