Documentation

Monlib.LinearAlgebra.QuantumSet.Instances

noncomputable def sig {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} (hφ : φ.IsFaithfulPosMap) (z : ) :
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem sig_apply {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} (hφ : φ.IsFaithfulPosMap) (z : ) (a : Matrix n n ) :
    (sig z) a = .rpow (-z) * a * .rpow z
    @[simp]
    theorem sig_symm_apply {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} (hφ : φ.IsFaithfulPosMap) (z : ) (a : Matrix n n ) :
    (sig z).symm a = .rpow z * a * .rpow (-z)
    theorem Module.Dual.IsFaithfulPosMap.sig_trans_sig {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] (x : ) (y : ) :
    (sig x).trans (sig y) = sig (x + y)
    theorem PosDef.smul {n : Type u_1} [Fintype n] {𝕜 : Type u_2} [RCLike 𝕜] {x : Matrix n n 𝕜} (hx : x.PosDef) (α : NNRealˣ) :
    (α x).PosDef
    theorem posSemidefOne_smul_rpow {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] (α : NNReal) (r : ) :
    .rpow r = (α ^ r) 1
    theorem posDefOne_smul_rpow {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] (α : NNRealˣ) (r : ) :
    .rpow r = (α ^ r) 1
    theorem Module.Dual.IsFaithfulPosMap.sig_zero {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] :
    sig 0 = 1
    theorem AlgEquiv.apply_eq_id {R : Type u_2} {M : Type u_3} [CommSemiring R] [Semiring M] [Algebra R M] {f : M ≃ₐ[R] M} :
    (∀ (x : M), f x = x) f = 1
    theorem Matrix.PosDef.rpow_neg_eq_inv_rpow {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] {Q : Matrix n n 𝕜} (hQ : Q.PosDef) (r : ) :
    hQ.rpow (-r) = (hQ.rpow r)⁻¹
    theorem RCLike.pos_toNNReal_units {𝕜 : Type u_2} [RCLike 𝕜] (r : 𝕜) :
    0 < r ∃ (s : NNRealˣ), r = s
    theorem RCLike.nonneg_toNNReal {𝕜 : Type u_2} [RCLike 𝕜] (r : 𝕜) :
    0 r ∃ (s : NNReal), r = s
    theorem Matrix.smulPosDef_isPosDef_iff {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] [H : Nonempty n] {Q : Matrix n n 𝕜} (hQ : Q.PosDef) (r : 𝕜) :
    (r Q).PosDef 0 < r
    theorem smul_onePosDef_rpow_eq {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] {α : 𝕜} (h : (α 1).PosDef) (r : ) :
    h.rpow r = (RCLike.re α ^ r) 1
    theorem Matrix.smulPosSemidef_isPosSemidef_iff {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] {Q : Matrix n n 𝕜} (hQ : Q.PosSemidef) (r : 𝕜) :
    (r Q).PosSemidef 0 r Q = 0
    theorem smul_onePosSemidef_rpow_eq {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] {α : 𝕜} (h : (α 1).PosSemidef) (r : ) :
    h.rpow r = (RCLike.re α ^ r) 1
    theorem Matrix.smul_one_inv {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] {s : NNRealˣ} :
    (s 1)⁻¹ = (↑s)⁻¹ 1
    theorem Matrix.PosDef.commutes_iff_rpow_commutes {𝕜 : Type u_2} [RCLike 𝕜] {n : Type u_3} [Fintype n] [DecidableEq n] {Q : Matrix n n 𝕜} (hQ : Q.PosDef) (r : ˣ) :
    (∀ (x : Matrix n n 𝕜), Commute x (hQ.rpow r)) ∀ (x : Matrix n n 𝕜), Commute x Q
    theorem Module.Dual.IsPosMap.isTracial_iff {n : Type u_2} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} (hφ : φ.IsPosMap) :
    φ.IsTracial ∃ (α : ), φ.matrix = α 1
    theorem sig_eq_id_iff {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] (k : ) :
    sig k = 1 k = 0 φ.IsTracial

    σ_k = 1 iff either k = 0 or φ is tracial

    theorem Module.Dual.pi_isTracial_iff {k : Type u_2} [Fintype k] [DecidableEq k] {s : kType u_3} [(i : k) → Fintype (s i)] [(i : k) → DecidableEq (s i)] {φ : (i : k) → Module.Dual (Matrix (s i) (s i) )} :
    (Module.Dual.pi φ).IsTracial ∀ (i : k), (φ i).IsTracial
    @[defaultInstance 1000]
    noncomputable instance Matrix.isStarAlgebra {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] :
    Equations
    noncomputable instance Module.Dual.IsFaithfulPosMap.innerProductAlgebra {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] :
    Equations
    noncomputable instance Module.Dual.IsFaithfulPosMap.quantumSet {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] :
    Equations
    • Module.Dual.IsFaithfulPosMap.quantumSet = QuantumSet.mk 0 (n × n) inferInstance inferInstance .orthonormalBasis
    noncomputable instance PiMat.isStarAlgebra {k : Type u_2} [Fintype k] {s : kType u_3} [(i : k) → Fintype (s i)] [(i : k) → DecidableEq (s i)] {ψ : (i : k) → Module.Dual (Matrix (s i) (s i) )} [_hψ : ∀ (i : k), (ψ i).IsFaithfulPosMap] :
    Equations
    • PiMat.isStarAlgebra = piStarAlgebra
    noncomputable instance Module.Dual.pi.IsFaithfulPosMap.innerProductAlgebra {k : Type u_2} [Fintype k] {s : kType u_3} [(i : k) → Fintype (s i)] [(i : k) → DecidableEq (s i)] {ψ : (i : k) → Module.Dual (Matrix (s i) (s i) )} [∀ (i : k), (ψ i).IsFaithfulPosMap] :
    Equations
    • Module.Dual.pi.IsFaithfulPosMap.innerProductAlgebra = piInnerProductAlgebra
    noncomputable instance Module.Dual.pi.IsFaithfulPosMap.quantumSet {k : Type u_2} [Fintype k] [DecidableEq k] {s : kType u_3} [(i : k) → Fintype (s i)] [(i : k) → DecidableEq (s i)] {ψ : (i : k) → Module.Dual (Matrix (s i) (s i) )} [hψ : ∀ (i : k), (ψ i).IsFaithfulPosMap] :
    Equations
    theorem LinearMap.mul'_comp_mul'_adjoint_of_delta_form {n : Type u_1} [Fintype n] [DecidableEq n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] :
    LinearMap.mul' (Matrix n n ) ∘ₗ Coalgebra.comul = φ.matrix⁻¹.trace 1
    theorem LinearMap.pi_mul'_comp_mul'_adjoint_of_delta_form {k : Type u_2} [Fintype k] [DecidableEq k] {s : kType u_3} [(i : k) → Fintype (s i)] [(i : k) → DecidableEq (s i)] [∀ (i : k), Nontrivial (s i)] {δ : } {φ : (i : k) → Module.Dual (Matrix (s i) (s i) )} [hφ : ∀ (i : k), (φ i).IsFaithfulPosMap] (hφ₂ : ∀ (i : k), (φ i).matrix⁻¹.trace = δ) :
    LinearMap.mul' (PiMat k s) ∘ₗ Coalgebra.comul = δ 1
    theorem Qam.Nontracial.delta_pos {n : Type u_1} [Fintype n] [DecidableEq n] [Nonempty n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] :
    0 < φ.matrix⁻¹.trace
    theorem Pi.Qam.Nontracial.delta_ne_zero {k : Type u_2} {s : kType u_3} [(i : k) → Fintype (s i)] [(i : k) → DecidableEq (s i)] [Nonempty k] [∀ (i : k), Nontrivial (s i)] {δ : } {φ : (i : k) → Module.Dual (Matrix (s i) (s i) )} [hφ : ∀ (i : k), (φ i).IsFaithfulPosMap] (hφ₂ : ∀ (i : k), (φ i).matrix⁻¹.trace = δ) :
    0 < δ
    noncomputable instance Matrix.quantumSetDeltaForm {n : Type u_1} [Fintype n] [DecidableEq n] [Nonempty n] {φ : Module.Dual (Matrix n n )} [hφ : φ.IsFaithfulPosMap] :
    Equations
    • Matrix.quantumSetDeltaForm = { delta := φ.matrix⁻¹.trace, delta_pos := , mul_comp_comul_eq := }
    noncomputable instance PiMat.quantumSetDeltaForm {k : Type u_2} [Fintype k] [DecidableEq k] {s : kType u_3} [(i : k) → Fintype (s i)] [(i : k) → DecidableEq (s i)] [Nonempty k] [∀ (i : k), Nontrivial (s i)] {d : } {φ : (i : k) → Module.Dual (Matrix (s i) (s i) )} [hφ : ∀ (i : k), (φ i).IsFaithfulPosMap] [hφ₂ : Fact (∀ (i : k), (φ i).matrix⁻¹.trace = d)] :
    Equations
    • PiMat.quantumSetDeltaForm = { delta := d, delta_pos := , mul_comp_comul_eq := }