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

@ -11,7 +11,6 @@ import Mathlib.Analysis.InnerProductSpace.PiL2
/-!
# The group SO(3)
-/
namespace GroupTheory
@ -107,7 +106,6 @@ lemma toProd_continuous : Continuous toProd := by
refine Continuous.matrix_transpose ?_
exact continuous_iff_le_induced.mpr fun U a => a
/-- The embedding of `SO(3)` into the monoid of matrices times the opposite of
the monoid of matrices. -/
lemma toProd_embedding : Embedding toProd where
@ -223,10 +221,7 @@ lemma exists_basis_preserved (A : SO(3)) :
use b
rw [hb, hv.2]
end action
end SO3
end GroupTheory