Zulip Chat Archive

Stream: Is there code for X?

Topic: Complexification of a real vector space


Arien Malec (Dec 13 2023 at 18:30):

I assume this (Exercise 1B Problem 7) from Axler's Linear Algebra is a one liner in Mathlib, but what one liner is it?

Suppose 𝑉 is a real vector space.
β€’ The complexification of 𝑉, denoted by 𝑉𝐂 , equals 𝑉 Γ— 𝑉. An element of
𝑉𝐂 is an ordered pair( 𝑒,𝑣),where𝑒,𝑣 ∈ 𝑉, but we write this as 𝑒+𝑖𝑣.
β€’ Addition on 𝑉𝐂 is defined by
(𝑒1 +𝑖𝑣1)+(𝑒2 +𝑖𝑣2) = (𝑒1 +𝑒2)+𝑖(𝑣1 +𝑣2) for all 𝑒1,𝑣1,𝑒2,𝑣2 βˆˆπ‘‰.
β€’ Complex scalar multiplication on 𝑉𝐂 is defined by (π‘Ž+𝑏𝑖)(𝑒+𝑖𝑣) = (π‘Žπ‘’βˆ’π‘π‘£)+𝑖(π‘Žπ‘£+𝑏𝑒)
for all π‘Ž, 𝑏 ∈ 𝐑 and all 𝑒, 𝑣 ∈ 𝑉.
Prove that with the definitions of addition and scalar multiplication as above,
𝑉𝐂 is a complex vector space.

Eric Rodriguez (Dec 13 2023 at 18:48):

This will be done with the tensor product in mathlib

Arien Malec (Dec 13 2023 at 19:26):

Something like:

variable [Module ℝ V]
#synth Module ℝ (TensorProduct ℝ V V)

?

Eric Wieser (Dec 13 2023 at 20:07):

No, more like:

import Mathlib

variable {V} [AddCommGroup V] [Module ℝ V]
open scoped TensorProduct

#synth Module β„‚ (β„‚ βŠ—[ℝ] V)

Eric Wieser (Dec 13 2023 at 20:12):

You can then prove your first bullet point as

def prodEquivComplexTensor : V Γ— V ≃ β„‚ βŠ—[ℝ] V := sorry

and the second one as

theorem smul_def (c : β„‚) (a : V Γ— V) :
    c β€’ prodEquivComplexTensor b = prodEquivComplexTensor (c.re β€’ a.1 - c.im β€’ a.2, c.re β€’ a.1 + c.im β€’ a.2) := by
  sorry

Arien Malec (Dec 17 2023 at 02:58):

I've been beating my head against the first theorem without seeing any cracks in the armor -- any Mathlib theorems that simply or open up the proof.

Richard Copley (Dec 17 2023 at 03:35):

TensorProduct.prodLeft or TensorProduct.prodRight should help.

Arien Malec (Dec 17 2023 at 04:46):

I'm having trouble getting the right types in place.... prodLeft wants to distribute a product over a tensor product.

Richard Copley (Dec 17 2023 at 05:03):

Can you show β„‚ ≃ₗ[R] (ℝ Γ— ℝ)? (It's hard to guess exactly how far you've got.)

Arien Malec (Dec 17 2023 at 05:03):

huh... Nice idea...

Arien Malec (Dec 17 2023 at 05:05):

You can assume that I've been searching for relating things in Mathlib and trying to see if I can find a chain of structural decomposition to force fit.

Richard Copley (Dec 17 2023 at 05:08):

Then there's TensorProduct.rid and TensorProduct.lid.


Last updated: Dec 20 2023 at 11:08 UTC