Zulip Chat Archive

Stream: maths

Topic: Unitary is not linear?


Bjørn Kjos-Hanssen (Sep 02 2022 at 00:26):

This seems strange:

import data.complex.basic
import algebra.star.unitary
theorem mwe (A:)(h:A  unitary ()) : ((star A) * A) 0 = 1 :=
calc (star A * A) 0 = (1:) 0: by rw h.1
                ... = 1: rfl

I would have expected (star A) * A to be the identity map?

Frédéric Dupuis (Sep 02 2022 at 00:38):

You're probably looking for ℂ →L[ℂ] ℂ instead of ℂ → ℂ. The monoid instance on ℂ → ℂ is docs#pi.monoid, which defines one to be λ x, 1, as you can see by trying

theorem mwe2 : (1 :   ) = λ x, 1 := rfl

Bjørn Kjos-Hanssen (Sep 02 2022 at 01:07):

Ah, thanks @Frédéric Dupuis . I guess it does make sense that in the general case of A:MNA: M \to N for monoids MNM\ne N, there is no identity map, so 1 should mean the constant function 1.

Bjørn Kjos-Hanssen (Sep 02 2022 at 01:15):

How do you type / import the L?

Jireh Loreaux (Sep 02 2022 at 01:17):

that's docs#continuous_linear_map. So anything that imports that will suffice.

Eric Wieser (Sep 02 2022 at 20:21):

You can also use 1 : function.End ℂ

Bjørn Kjos-Hanssen (Sep 02 2022 at 21:06):

Thanks @Eric Wieser Indeed, I was wondering if there was a way to take advantage of the fact that an identity function exists when M=NM=N (above)

Bjørn Kjos-Hanssen (Sep 02 2022 at 21:07):

To guarantee that unitary maps are linear perhaps we have to use something like euclidean_space?

Notification Bot (Sep 02 2022 at 21:07):

Bjørn Kjos-Hanssen has marked this topic as unresolved.

Kevin Buzzard (Sep 02 2022 at 22:11):

The identity function M -> M is called id rather than 1.

Jireh Loreaux (Sep 04 2022 at 04:51):

docs#unitary is a submonoid of a star monoid. That is, for any type with star, 1 and * (plus compatibility requirements), the unitary elements are exactly those u such that u⁻¹ = u⋆. So, for example, u : unitary ℂ is a complex number of modulus one. One can always view unitaries as elements of the original monoid (i.e., if u : unitary ℂ, then ↑u : ℂ makes sense, the is a coercion). However, there is no way to view this as a linear map; I know there is mathematically, but there is no linear coercion from to linear maps from to . Thus, in general, one cannot think of unitaries as linear maps.

Note that this is what you should expect. For example, if A is a C⋆-algebra, and u : unitary A, then it makes sense to think of ↑u : A, but the only way to think of u as a linear map is to represent A faithfully on some Hilbert space, but which one should you choose? So, we shouldn't expect this behavior.

Finally, to answer what I think is your question: the type of linear maps E →ₗ[𝕜] E where E is an inner product space over 𝕜 (= or ) has an docs#linear_map.adjoint which is the docs#linear_map.has_star operation on this type. Moreover, such linear maps also have 1 and * (identity map and composition). Therefore, unitary (E →ₗ[𝕜] E) makes sense and some u of this type will have a coercion to an honest-to-God linear map.

Jireh Loreaux (Sep 04 2022 at 04:54):

The type euclidean_space ℂ (fin n) →ₗ[ℂ] euclidean_space ℂ (fin n) where n : ℕ is the type of all -linear maps from ℂⁿ to itself.


Last updated: Dec 20 2023 at 11:08 UTC