Zulip Chat Archive

Stream: maths

Topic: Antilinear functions over the reals


Daniel Roca González (Jan 15 2022 at 20:23):

Hello everyone,
I'm working over a real Hilbert space E and want to use the Riesz representation lemma. inner_product_space.to_dual from mathlib gives me an equivalence E ≃ₛₗᵢ[↑conj] normed_space.dual 𝕜 E, from which one can get an antilinear map normed_space.dual ℝ E →ₛₗ[↑conj] E. How can I get a linear map from this? I'm not sure how to begin...

Heather Macbeth (Jan 15 2022 at 20:31):

@Daniel Roca González It is designed to "just work". An antilinear map over is definitionally a linear map.

Heather Macbeth (Jan 15 2022 at 20:33):

import analysis.inner_product_space.dual

noncomputable theory

variables {E : Type*} [inner_product_space  E] [complete_space E]

example : E ≃ₗᵢ[] normed_space.dual  E := inner_product_space.to_dual  E

Daniel Roca González (Jan 15 2022 at 20:41):

wow I can't believe I didn't try this, thank you. Yeah this works just fine.

Heather Macbeth (Jan 15 2022 at 20:42):

If you'd like to know more:
https://leanprover-community.github.io/blog/posts/semilinear-maps/

Daniel Roca González (Jan 15 2022 at 20:55):

Thanks a lot. I think I had understood that linear maps are defined as semilinear maps, but I somehow didn't make the connection that ↑conj is equal to the identity definitionally


Last updated: Dec 20 2023 at 11:08 UTC