Skip to content

Commit fb9a612

Browse files
chore: simplify variables in LinearAlgebra.Dimension.Torsion.Finite (#19839)
1 parent d1e3519 commit fb9a612

File tree

1 file changed

+3
-18
lines changed

1 file changed

+3
-18
lines changed

Mathlib/LinearAlgebra/Dimension/Torsion/Finite.lean

Lines changed: 3 additions & 18 deletions
Original file line numberDiff line numberDiff line change
@@ -11,29 +11,14 @@ import Mathlib.LinearAlgebra.Dimension.Finite
1111
1212
-/
1313

14-
universe u v
14+
variable {R M : Type*} [CommRing R] [IsDomain R] [AddCommGroup M] [Module R M]
1515

16-
variable {R : Type u} {M : Type v}
17-
variable [Ring R] [AddCommGroup M]
18-
19-
section RankZero
20-
21-
variable [Nontrivial R]
22-
23-
lemma rank_eq_zero_iff_isTorsion {R M} [CommRing R] [IsDomain R] [AddCommGroup M] [Module R M] :
24-
Module.rank R M = 0 ↔ Module.IsTorsion R M := by
16+
lemma rank_eq_zero_iff_isTorsion: Module.rank R M = 0 ↔ Module.IsTorsion R M := by
2517
rw [Module.IsTorsion, rank_eq_zero_iff]
2618
simp [mem_nonZeroDivisors_iff_ne_zero]
2719

28-
end RankZero
29-
30-
section StrongRankCondition
31-
3220
/-- The `StrongRankCondition` is automatic. See `commRing_strongRankCondition`. -/
33-
theorem Module.finrank_eq_zero_iff_isTorsion {R} [CommRing R] [StrongRankCondition R]
34-
[IsDomain R] [Module R M] [Module.Finite R M] :
21+
theorem Module.finrank_eq_zero_iff_isTorsion [StrongRankCondition R] [Module.Finite R M] :
3522
finrank R M = 0 ↔ Module.IsTorsion R M := by
3623
rw [← rank_eq_zero_iff_isTorsion (R := R), ← finrank_eq_rank]
3724
norm_cast
38-
39-
end StrongRankCondition

0 commit comments

Comments
 (0)