Skip to content

Commit

Permalink
chore: rename star_mul_self_nonneg' (#8305)
Browse files Browse the repository at this point in the history
  • Loading branch information
j-loreaux committed Nov 10, 2023
1 parent 1d77564 commit 7a1bf93
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Star/Order.lean
Original file line number Diff line number Diff line change
Expand Up @@ -152,9 +152,9 @@ theorem star_mul_self_nonneg (r : R) : 0 ≤ star r * r :=
StarOrderedRing.nonneg_iff.mpr <| AddSubmonoid.subset_closure ⟨r, rfl⟩
#align star_mul_self_nonneg star_mul_self_nonneg

theorem star_mul_self_nonneg' (r : R) : 0 ≤ r * star r := by
theorem mul_star_self_nonneg (r : R) : 0 ≤ r * star r := by
simpa only [star_star] using star_mul_self_nonneg (star r)
#align star_mul_self_nonneg' star_mul_self_nonneg'
#align star_mul_self_nonneg' mul_star_self_nonneg

theorem conjugate_nonneg {a : R} (ha : 0 ≤ a) (c : R) : 0 ≤ star c * a * c := by
rw [StarOrderedRing.nonneg_iff] at ha
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/Matrix/DotProduct.lean
Original file line number Diff line number Diff line change
Expand Up @@ -94,7 +94,7 @@ theorem dotProduct_star_self_eq_zero {v : n → R} : dotProduct (star v) v = 0
/-- Note that this applies to `ℂ` via `Complex.strictOrderedCommRing`. -/
@[simp]
theorem dotProduct_self_star_eq_zero {v : n → R} : dotProduct v (star v) = 0 ↔ v = 0 :=
(Finset.sum_eq_zero_iff_of_nonneg fun i _ => (@star_mul_self_nonneg' _ _ _ _ (v i) : _)).trans <|
(Finset.sum_eq_zero_iff_of_nonneg fun i _ => (@mul_star_self_nonneg _ _ _ _ (v i) : _)).trans <|
by simp [Function.funext_iff, mul_eq_zero]
#align matrix.dot_product_self_star_eq_zero Matrix.dotProduct_self_star_eq_zero

Expand Down

0 comments on commit 7a1bf93

Please sign in to comment.