Skip to content

Commit 68b69b5

Browse files
committed
comment + finrank version
1 parent 3ffa427 commit 68b69b5

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

Mathlib/LinearAlgebra/Dimension/Basic.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -229,6 +229,11 @@ theorem rank_eq_of_equiv_equiv (i : R → R') (j : M ≃+ M₁)
229229
end
230230
end Semiring
231231

232+
/-- TODO: prove that nontrivial commutative semirings satisfy the strong rank condition,
233+
following *Free sets and free subsemimodules in a semimodule* by Yi-Jia Tan, Theorem 3.2.
234+
235+
Rings `R` that fail the strong rank condition but satisfy `rank R R = 1` are expected to exist, see
236+
https://mathoverflow.net/questions/317422/rings-that-fail-to-satisfy-the-strong-rank-condition. -/
232237
theorem CommSemiring.rank_self (R) [CommSemiring R] : Module.rank R R = 1 := by
233238
nontriviality R
234239
rw [le_antisymm_iff, ← not_lt, ← Order.succ_le_iff, ← Nat.cast_one, ← nat_succ,
@@ -240,6 +245,9 @@ theorem CommSemiring.rank_self (R) [CommSemiring R] : Module.rank R R = 1 := by
240245
have h₂ : 0 = f ![1, 0] := by simpa using congr($this 1)
241246
exact zero_ne_one (α := R) (by simpa using congr($(inj (h₁.trans h₂)) 1))
242247

248+
theorem CommSemiring.finrank_self (R) [CommSemiring R] : Module.finrank R R = 1 :=
249+
Module.finrank_eq_of_rank_eq (rank_self R)
250+
243251
section Ring
244252
variable [Ring R] [AddCommGroup M] [Module R M] [Ring R']
245253

0 commit comments

Comments
 (0)