Skip to content

Commit

Permalink
Update NoZeroSMulDivisors.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
syur2 committed Oct 19, 2024
1 parent 4b5edb2 commit f60fcd9
Showing 1 changed file with 19 additions and 6 deletions.
25 changes: 19 additions & 6 deletions ModuleLocalProperties/NoZeroSMulDivisors.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,12 +11,6 @@ import ModuleLocalProperties.MissingLemmas.LocalizedModule

open Submodule LocalizedModule IsLocalizedModule LinearMap nonZeroDivisors

#check IsLocalization.map_comap
#check Module.annihilator
#check NoZeroSMulDivisors
#check IsLocalization.map_nonZeroDivisors_le
#check IsDomain

section missinglemma

lemma IsLocalization.mem_map_nonZeroDivisors {R : Type*} [CommSemiring R] (S : Submonoid R)
Expand Down Expand Up @@ -111,3 +105,22 @@ lemma localized_torsion [IsDomain R] :
exact localized_torsion_nontrival_ge _ _ trivial

end localized_torsion_commutivity

section NoZeroSMulDivisors_local_property

variable {R : Type*} [CommRing R] [IsDomain R] (M : Type*) [AddCommGroup M] [Module R M]

lemma noZeroSMulDivisors_of_localization (h : ∀ (J : Ideal R) (hJ : J.IsMaximal),

This comment has been minimized.

Copy link
@mbkybky

mbkybky Oct 19, 2024

Owner

I think maybe this theorem is true for all CommRing R.

NoZeroSMulDivisors (Localization J.primeCompl) (LocalizedModule J.primeCompl M)) :
NoZeroSMulDivisors R M :=
noZeroSMulDivisors_iff_torsion_eq_bot.mpr <| submodule_eq_bot_of_localization _ <| fun J hJ ↦
localized_torsion J.primeCompl M ▸ noZeroSMulDivisors_iff_torsion_eq_bot.mp <| h J hJ

lemma noZeroSMulDivisors_of_localization_iff :

This comment has been minimized.

Copy link
@mbkybky

mbkybky Oct 19, 2024

Owner

I think it is better to prove that if M is NoZeroSMulDivisors, then its localization is NoZeroSMulDivisors. And it is also true for all CommRing R.

NoZeroSMulDivisors R M ↔ ∀ (J : Ideal R) (hJ : J.IsMaximal),
NoZeroSMulDivisors (Localization J.primeCompl) (LocalizedModule J.primeCompl M) :=
fun h J _ ↦ (noZeroSMulDivisors_iff_torsion_eq_bot.mp h) ▸ localized_torsion J.primeCompl M ▸
noZeroSMulDivisors_iff_torsion_eq_bot.mpr <| localized_bot _ ,
fun h ↦ noZeroSMulDivisors_of_localization M h⟩

end NoZeroSMulDivisors_local_property

0 comments on commit f60fcd9

Please sign in to comment.