Update Rows.lean

This commit is contained in:
jstoobysmith 2024-11-02 07:57:22 +00:00
parent 3de17d1444
commit 2f2f2ff3d1

View file

@ -186,7 +186,7 @@ lemma rows_linearly_independent (V : CKMMatrix) : LinearIndependent (rows V)
· exact h1
· exact h2
lemma rows_card : Fintype.card (Fin 3) = FiniteDimensional.finrank (Fin 3 → ) := by
lemma rows_card : Fintype.card (Fin 3) = Module.finrank (Fin 3 → ) := by
simp
/-- The rows of a CKM matrix as a basis of `ℂ³`. -/