Skip to content

Commit

Permalink
chore(linear_algebra/quadratic_form): make Sylvester's law of inertia…
Browse files Browse the repository at this point in the history
… bold in the doc string (#8610)
  • Loading branch information
JasonKYi committed Aug 10, 2021
1 parent e2b7f70 commit 5739199
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/linear_algebra/quadratic_form.lean
Expand Up @@ -978,7 +978,7 @@ begin
apply_instance
end

/-- Sylvester's law of inertia: A nondegenerate real quadratic form is equivalent to a weighted
/-- **Sylvester's law of inertia**: A nondegenerate real quadratic form is equivalent to a weighted
sum of squares with the weights being ±1. -/
theorem equivalent_one_neg_one_weighted_sum_squared
{M : Type*} [add_comm_group M] [module ℝ M] [finite_dimensional ℝ M]
Expand Down

0 comments on commit 5739199

Please sign in to comment.