Skip to content

Commit c174b2d

Browse files
committed
chore(Module/Torsion): drop DecidableEq assumptions (#10253)
1 parent 8dd23a4 commit c174b2d

File tree

1 file changed

+4
-5
lines changed

1 file changed

+4
-5
lines changed

Mathlib/Algebra/Module/Torsion.lean

Lines changed: 4 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -392,7 +392,7 @@ variable {ι : Type*} {p : ι → Ideal R} {S : Finset ι}
392392
variable (hp : (S : Set ι).Pairwise fun i j => p i ⊔ p j = ⊤)
393393

394394
-- Porting note: mem_iSup_finset_iff_exists_sum now requires DecidableEq ι
395-
theorem iSup_torsionBySet_ideal_eq_torsionBySet_iInf [DecidableEq ι] :
395+
theorem iSup_torsionBySet_ideal_eq_torsionBySet_iInf :
396396
⨆ i ∈ S, torsionBySet R M (p i) = torsionBySet R M ↑(⨅ i ∈ S, p i) := by
397397
rcases S.eq_empty_or_nonempty with h | h
398398
· simp only [h]
@@ -430,7 +430,7 @@ theorem iSup_torsionBySet_ideal_eq_torsionBySet_iInf [DecidableEq ι] :
430430
#align submodule.supr_torsion_by_ideal_eq_torsion_by_infi Submodule.iSup_torsionBySet_ideal_eq_torsionBySet_iInf
431431

432432
-- Porting note: iSup_torsionBySet_ideal_eq_torsionBySet_iInf now requires DecidableEq ι
433-
theorem supIndep_torsionBySet_ideal [DecidableEq ι] : S.SupIndep fun i => torsionBySet R M <| p i :=
433+
theorem supIndep_torsionBySet_ideal : S.SupIndep fun i => torsionBySet R M <| p i :=
434434
fun T hT i hi hiT => by
435435
rw [disjoint_iff, Finset.sup_eq_iSup,
436436
iSup_torsionBySet_ideal_eq_torsionBySet_iInf fun i hi j hj ij => hp (hT hi) (hT hj) ij]
@@ -443,7 +443,7 @@ theorem supIndep_torsionBySet_ideal [DecidableEq ι] : S.SupIndep fun i => torsi
443443

444444
variable {q : ι → R} (hq : (S : Set ι).Pairwise <| (IsCoprime on q))
445445

446-
theorem iSup_torsionBy_eq_torsionBy_prod [DecidableEq ι] :
446+
theorem iSup_torsionBy_eq_torsionBy_prod :
447447
⨆ i ∈ S, torsionBy R M (q i) = torsionBy R M (∏ i in S, q i) := by
448448
rw [← torsionBySet_span_singleton_eq, Ideal.submodule_span_eq, ←
449449
Ideal.finset_inf_span_singleton _ _ hq, Finset.inf_eq_iInf, ←
@@ -456,8 +456,7 @@ theorem iSup_torsionBy_eq_torsionBy_prod [DecidableEq ι] :
456456
exact fun i hi j hj ij => (Ideal.sup_eq_top_iff_isCoprime _ _).mpr (hq hi hj ij)
457457
#align submodule.supr_torsion_by_eq_torsion_by_prod Submodule.iSup_torsionBy_eq_torsionBy_prod
458458

459-
-- Porting note: supIndep_torsionBySet_ideal now requires DecidableEq ι
460-
theorem supIndep_torsionBy [DecidableEq ι] : S.SupIndep fun i => torsionBy R M <| q i := by
459+
theorem supIndep_torsionBy : S.SupIndep fun i => torsionBy R M <| q i := by
461460
convert supIndep_torsionBySet_ideal (M := M) fun i hi j hj ij =>
462461
(Ideal.sup_eq_top_iff_isCoprime (q i) _).mpr <| hq hi hj ij
463462
exact (torsionBySet_span_singleton_eq (R := R) (M := M) _).symm

0 commit comments

Comments
 (0)