File tree Expand file tree Collapse file tree 1 file changed +3
-18
lines changed
Mathlib/LinearAlgebra/Dimension/Torsion Expand file tree Collapse file tree 1 file changed +3
-18
lines changed Original file line number Diff line number Diff line change @@ -11,29 +11,14 @@ import Mathlib.LinearAlgebra.Dimension.Finite
11
11
12
12
-/
13
13
14
- universe u v
14
+ variable {R M : Type *} [CommRing R] [IsDomain R] [AddCommGroup M] [Module R M]
15
15
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
25
17
rw [Module.IsTorsion, rank_eq_zero_iff]
26
18
simp [mem_nonZeroDivisors_iff_ne_zero]
27
19
28
- end RankZero
29
-
30
- section StrongRankCondition
31
-
32
20
/-- 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] :
35
22
finrank R M = 0 ↔ Module.IsTorsion R M := by
36
23
rw [← rank_eq_zero_iff_isTorsion (R := R), ← finrank_eq_rank]
37
24
norm_cast
38
-
39
- end StrongRankCondition
You can’t perform that action at this time.
0 commit comments