clean mathematics
This commit is contained in:
parent
fa425ef606
commit
d911b3b0f9
5 changed files with 9 additions and 9 deletions
|
@ -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
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue