Documentation

Monlib.LinearAlgebra.QuantumSet.SchurMul

Schur product operator #

In this file we define the Schur product operator and prove some basic properties.

noncomputable def schurMul {B : Type u_1} {C : Type u_2} [starAlgebra B] [starAlgebra C] [hB : QuantumSet B] [hC : QuantumSet C] :

Schur product ⬝ •ₛ ⬝ : (B → C) → (B → C) → (B → C) given by x •ₛ y := m ∘ (x ⊗ y) ∘ comul

Equations
  • One or more equations did not get rendered due to their size.
Instances For

    Schur product ⬝ •ₛ ⬝ : (B → C) → (B → C) → (B → C) given by x •ₛ y := m ∘ (x ⊗ y) ∘ comul

    Equations
    Instances For

      Pretty printer defined by notation3 command.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        theorem schurMul.apply_rankOne {B : Type u_1} {C : Type u_2} [starAlgebra B] [starAlgebra C] [hB : QuantumSet B] [hC : QuantumSet C] (a : B) (b : C) (c : B) (d : C) :
        (((rankOne ) a) b) •ₛ (((rankOne ) c) d) = (((rankOne ) (a * c)) (b * d))
        theorem schurMul.apply_ket {B : Type u_1} [starAlgebra B] [hB : QuantumSet B] (a b : B) :
        ((ket ) a) •ₛ ((ket ) b) = ((ket ) (a * b))
        theorem bra_tmul {𝕜 : Type u_1} {B : Type u_2} {C : Type u_3} [RCLike 𝕜] [NormedAddCommGroup B] [NormedAddCommGroup C] [InnerProductSpace 𝕜 B] [InnerProductSpace 𝕜 C] [FiniteDimensional 𝕜 B] [FiniteDimensional 𝕜 C] (a : B) (b : C) :
        ((bra 𝕜) (a ⊗ₜ[𝕜] b)) = (TensorProduct.lid 𝕜 𝕜) ∘ₗ TensorProduct.map ((bra 𝕜) a) ((bra 𝕜) b)
        theorem bra_map_bra {𝕜 : Type u_1} {B : Type u_2} {C : Type u_3} [RCLike 𝕜] [NormedAddCommGroup B] [NormedAddCommGroup C] [InnerProductSpace 𝕜 B] [InnerProductSpace 𝕜 C] [FiniteDimensional 𝕜 B] [FiniteDimensional 𝕜 C] (a : B) (b : C) :
        TensorProduct.map ((bra 𝕜) a) ((bra 𝕜) b) = (TensorProduct.lid 𝕜 𝕜).symm ∘ₗ ((bra 𝕜) (a ⊗ₜ[𝕜] b))
        theorem ket_tmul {𝕜 : Type u_1} {B : Type u_2} {C : Type u_3} [RCLike 𝕜] [NormedAddCommGroup B] [NormedAddCommGroup C] [InnerProductSpace 𝕜 B] [InnerProductSpace 𝕜 C] [FiniteDimensional 𝕜 B] [FiniteDimensional 𝕜 C] (a : B) (b : C) :
        ((ket 𝕜) (a ⊗ₜ[𝕜] b)) = TensorProduct.map ((ket 𝕜) a) ((ket 𝕜) b) ∘ₗ (TensorProduct.lid 𝕜 𝕜).symm
        theorem ket_map_ket {𝕜 : Type u_1} {B : Type u_2} {C : Type u_3} [RCLike 𝕜] [NormedAddCommGroup B] [NormedAddCommGroup C] [InnerProductSpace 𝕜 B] [InnerProductSpace 𝕜 C] [FiniteDimensional 𝕜 B] [FiniteDimensional 𝕜 C] (a : B) (b : C) :
        TensorProduct.map ((ket 𝕜) a) ((ket 𝕜) b) = ((ket 𝕜) (a ⊗ₜ[𝕜] b)) ∘ₗ (TensorProduct.lid 𝕜 𝕜)
        theorem rankOne_tmul {𝕜 : Type u_1} {B : Type u_2} {C : Type u_3} [RCLike 𝕜] [NormedAddCommGroup B] [NormedAddCommGroup C] [InnerProductSpace 𝕜 B] [InnerProductSpace 𝕜 C] [FiniteDimensional 𝕜 B] [FiniteDimensional 𝕜 C] {A : Type u_4} {D : Type u_5} [NormedAddCommGroup A] [NormedAddCommGroup D] [InnerProductSpace 𝕜 A] [InnerProductSpace 𝕜 D] [FiniteDimensional 𝕜 A] [FiniteDimensional 𝕜 D] (a : A) (b : B) (c : C) (d : D) :
        (((rankOne 𝕜) (a ⊗ₜ[𝕜] c)) (b ⊗ₜ[𝕜] d)) = TensorProduct.map (((rankOne 𝕜) a) b) (((rankOne 𝕜) c) d)
        theorem bra_comp_linearMap {𝕜 : Type u_1} {E₁ : Type u_2} {E₂ : Type u_3} [RCLike 𝕜] [NormedAddCommGroup E₁] [InnerProductSpace 𝕜 E₁] [NormedAddCommGroup E₂] [InnerProductSpace 𝕜 E₂] [FiniteDimensional 𝕜 E₁] [FiniteDimensional 𝕜 E₂] (x : E₂) (f : E₁ →ₗ[𝕜] E₂) :
        ((bra 𝕜) x) ∘ₗ f = ((bra 𝕜) ((LinearMap.adjoint f) x))
        theorem linearMap_comp_ket {𝕜 : Type u_1} {E₁ : Type u_2} {E₂ : Type u_3} [RCLike 𝕜] [NormedAddCommGroup E₁] [InnerProductSpace 𝕜 E₁] [NormedAddCommGroup E₂] [InnerProductSpace 𝕜 E₂] (x : E₁) (f : E₁ →ₗ[𝕜] E₂) :
        f ∘ₗ ((ket 𝕜) x) = ((ket 𝕜) (f x))
        theorem schurMul.apply_bra {B : Type u_1} [starAlgebra B] [hB : QuantumSet B] (a b : B) :
        ((bra ) a) •ₛ ((bra ) b) = ((bra ) (a * b))
        theorem schurMul.comp_apply_of {A : Type u_1} {B : Type u_3} {C : Type u_5} [starAlgebra A] [starAlgebra B] [starAlgebra C] [hA : QuantumSet A] [hB : QuantumSet B] [hC : QuantumSet C] (δ : ) (hAδ : CoalgebraStruct.comul ∘ₗ LinearMap.mul' A = δ LinearMap.id) (a b : A →ₗ[] B) (c d : C →ₗ[] A) :
        (a •ₛ b) ∘ₗ c •ₛ d = δ (a ∘ₗ c) •ₛ b ∘ₗ d
        theorem schurMul_one_one_right {B : Type u_2} {C : Type u_1} [starAlgebra B] [starAlgebra C] [hB : QuantumSet B] [hC : QuantumSet C] (A : C →ₗ[] B) :
        A •ₛ (((rankOne ) 1) 1) = A
        theorem schurMul_one_one_left {B : Type u_2} {C : Type u_1} [starAlgebra B] [starAlgebra C] [hB : QuantumSet B] [hC : QuantumSet C] (A : C →ₗ[] B) :
        (((rankOne ) 1) 1) •ₛ A = A
        theorem schurMul_real {A : Type u_1} {B : Type u_2} [starAlgebra A] [starAlgebra B] [hA : QuantumSet A] [hB : QuantumSet B] (x y : A →ₗ[] B) :
        theorem schurMul_one_right_rankOne {B : Type u_1} [starAlgebra B] [hB : QuantumSet B] (a b : B) :
        theorem schurMul_one_left_rankOne {B : Type u_1} [starAlgebra B] [hB : QuantumSet B] (a b : B) :
        theorem Psi.schurMul {A : Type u_1} {B : Type u_2} [starAlgebra A] [starAlgebra B] [hA : QuantumSet A] [hB : QuantumSet B] (r₁ r₂ : ) (f g : A →ₗ[] B) :
        (QuantumSet.Psi r₁ r₂) (f •ₛ g) = (QuantumSet.Psi r₁ r₂) f * (QuantumSet.Psi r₁ r₂) g
        theorem schurMul_assoc {A : Type u_1} {B : Type u_2} [starAlgebra A] [starAlgebra B] [hA : QuantumSet A] [hB : QuantumSet B] (f g h : A →ₗ[] B) :
        (f •ₛ g) •ₛ h = f •ₛ g •ₛ h
        theorem schurMul_one_iff_one_schurMul_of_isReal {A : Type u_1} {B : Type u_2} [starAlgebra A] [starAlgebra B] [hA : QuantumSet A] [hB : QuantumSet B] {x y z : A →ₗ[] B} (hx : LinearMap.IsReal x) (hy : LinearMap.IsReal y) (hz : LinearMap.IsReal z) :
        x •ₛ y = z y •ₛ x = z
        theorem schurMul_reflexive_of_isReal {A : Type u_1} [starAlgebra A] [hA : QuantumSet A] {x : A →ₗ[] A} (hx : LinearMap.IsReal x) :
        x •ₛ 1 = 1 1 •ₛ x = 1
        theorem schurMul_irreflexive_of_isReal {A : Type u_1} [starAlgebra A] [hA : QuantumSet A] {x : A →ₗ[] A} (hx : LinearMap.IsReal x) :
        x •ₛ 1 = 0 1 •ₛ x = 0