Skip to content

Commit

Permalink
remove gns/kms in QuantumGraph.Degree
Browse files Browse the repository at this point in the history
  • Loading branch information
themathqueen committed Nov 14, 2024
1 parent 7e5e06c commit 5beb572
Show file tree
Hide file tree
Showing 2 changed files with 462 additions and 14 deletions.
6 changes: 3 additions & 3 deletions Monlib/LinearAlgebra/Matrix/PosEqLinearMapIsPositive.lean
Original file line number Diff line number Diff line change
Expand Up @@ -273,7 +273,7 @@ theorem Matrix.posSemidef_iff_eq_rankOne' [Fintype n] [DecidableEq n] {x : Matri
Matrix.posSemidef_iff_eq_rankOne
theorem Matrix.posSemidef_iff_eq_rankOne'' [Fintype n] [DecidableEq n] {x : Matrix n n π•œ} :
x.PosSemidef ↔
βˆƒ (m : Type) (hm : Fintype m) (v : m β†’ (n β†’ π•œ)),
βˆƒ (m : Type) (_hm : Fintype m) (v : m β†’ (n β†’ π•œ)),
x =
βˆ‘ i : m,
LinearMap.toMatrix' (rankOne π•œ ((EuclideanSpace.equiv _ _).symm (v i)) ((EuclideanSpace.equiv _ _).symm (v i))).toLinearMap :=
Expand Down Expand Up @@ -329,7 +329,7 @@ theorem Matrix.posSemidef_iff_col_mul_conjTranspose_col [Fintype n] [DecidableEq
simp_rw [Matrix.posSemidef_iff_eq_rankOne, rankOne.EuclideanSpace.toMatrix']
theorem Matrix.posSemidef_iff_col_mul_conjTranspose_col' [Fintype n] [DecidableEq n] {x : Matrix n n π•œ} :
x.PosSemidef ↔
βˆƒ (m : Type) (hm : Fintype m) (v : m β†’ EuclideanSpace π•œ n),
βˆƒ (m : Type) (_hm : Fintype m) (v : m β†’ EuclideanSpace π•œ n),
x =
βˆ‘ i : m, col (Fin 1) (v i : n β†’ π•œ) * (col (Fin 1) (v i : n β†’ π•œ))α΄΄ :=
by
Expand All @@ -341,7 +341,7 @@ theorem Matrix.posSemidef_iff_vecMulVec [Fintype n] [DecidableEq n] {x : Matrix
x = βˆ‘ i : Fin m, vecMulVec (v i) (star (v i)) :=
by simp_rw [Matrix.posSemidef_iff_col_mul_conjTranspose_col, vecMulVec_eq (Fin 1), conjTranspose_col]
theorem Matrix.posSemidef_iff_vecMulVec' [Fintype n] [DecidableEq n] {x : Matrix n n π•œ} :
x.PosSemidef ↔ βˆƒ (m : Type) (hm : Fintype m) (v : m β†’ EuclideanSpace π•œ n),
x.PosSemidef ↔ βˆƒ (m : Type) (_hm : Fintype m) (v : m β†’ EuclideanSpace π•œ n),
x = βˆ‘ i : m, vecMulVec (v i) (star (v i)) :=
by simp_rw [Matrix.posSemidef_iff_col_mul_conjTranspose_col', vecMulVec_eq (Fin 1), conjTranspose_col]

Expand Down
Loading

0 comments on commit 5beb572

Please sign in to comment.