Zulip Chat Archive

Stream: maths

Topic: Determinant of an element of orthogonal/unitary groups


Heather Macbeth (Jun 14 2021 at 17:44):

Since #7635 (@Anne Baanen) it is possible to state that the determinant of an isometry has absolute value 1:

import analysis.normed_space.inner_product
import linear_algebra.determinant

variables (๐•œ : Type*) [is_R_or_C ๐•œ]
variables {E : Type*} [inner_product_space ๐•œ E] [finite_dimensional ๐•œ E]

open is_R_or_C

lemma linear_isometry.abs_det (f : E โ†’โ‚—แตข[๐•œ] E) : abs f.to_linear_map.det = 1 := sorry

Is this on someone's to-do list? How should it even be proved? (Since mathlib doesn't have the adjoint construction ... the conjugate linear map problem again.)


Last updated: Dec 20 2023 at 11:08 UTC