Zulip Chat Archive

Stream: Is there code for X?

Topic: module finite if localizations are finite


Christian Merten (Jun 23 2024 at 09:38):

Do we have something like:

import Mathlib

theorem finite_ofLocalizationSpanTarget {R M : Type*} [CommRing R] [AddCommMonoid M]
    [Module R M] (t : Finset R) (ht : Ideal.span (t : Set R) = )
    (H :  (g : t), Module.Finite (Localization.Away g.val)
      (LocalizedModule (Submonoid.powers g.val) M)) :
    Module.Finite R M := by
  sorry

Probably @Andrew Yang knows this?

Andrew Yang (Jun 23 2024 at 09:43):

We have docs#finite_ofLocalizationSpan, but I'm not sure how easy it is to massage it into this.

Christian Merten (Jun 23 2024 at 09:45):

Ah thanks, I was looking in RingTheory/RingHom/Finite.

Christian Merten (Jun 23 2024 at 09:54):

To mimic docs#finite_ofLocalizationSpan, I probably have to mimic docs#IsLocalization.finsetIntegerMultiple first.

Andrew Yang (Jun 23 2024 at 10:14):

Yeah we should move them into RingTheory/RingHom/Finite.

Andrew Yang (Jun 23 2024 at 10:14):

It should follow easily once the localisation refactors land, but currently they are a performance hazard and I've yet to try all the suggestions by Matthew.

Christian Merten (Jun 23 2024 at 10:17):

Andrew Yang said:

It should follow easily once the localisation refactors land, but currently they are a performance hazard and I've yet to try all the suggestions by Matthew.

To unxy: This is the last step to show that finite presentation is a local ring hom property. So I think I'll try to finish it for the time being.

Andrew Yang (Jun 23 2024 at 10:20):

Sounds good!
In case it wasn't clear, that comment wasn't meant to block new development, and instead just another reason for me to resume the refactor work.


Last updated: May 02 2025 at 03:31 UTC