refactor: Remove double empty lines

This commit is contained in:
jstoobysmith 2024-07-03 07:56:30 -04:00
parent ae18a2196d
commit f03d063c86
60 changed files with 0 additions and 232 deletions

View file

@ -58,7 +58,6 @@ lemma exists_plane_exists_basis {n : } (hE : ExistsPlane n) :
| Sum.inl i => exact h3 i
| Sum.inr i => exact h4 i
theorem plane_exists_dim_le_7 {n : } (hn : ExistsPlane n) : n ≤ 7 := by
obtain ⟨B, hB⟩ := exists_plane_exists_basis hn
have h1 := LinearIndependent.fintype_card_le_finrank hB
@ -67,6 +66,5 @@ theorem plane_exists_dim_le_7 {n : } (hn : ExistsPlane n) : n ≤ 7 := by
FiniteDimensional.finrank_fin_fun ] at h1
exact Nat.le_of_add_le_add_left h1
end PlusU1
end SMRHN