clean mathematics

This commit is contained in:
Pietro Monticone 2025-01-14 00:11:17 +01:00
parent fa425ef606
commit d911b3b0f9
5 changed files with 9 additions and 9 deletions

View file

@ -57,7 +57,7 @@ lemma subtype_val_eq_toGL : (Subtype.val : SO3 → Matrix (Fin 3) (Fin 3) ) =
Units.val ∘ toGL.toFun :=
rfl
/-- The inclusino of `SO(3)` into `GL(3,)` is an injection. -/
/-- The inclusion of `SO(3)` into `GL(3,)` is an injection. -/
lemma toGL_injective : Function.Injective toGL := by
refine fun A B h ↦ Subtype.eq ?_
rw [@Units.ext_iff] at h