Skip to content

Commit

Permalink
feat(linear_algebra/quadratic_form): add associated_eq_self_apply (#6458
Browse files Browse the repository at this point in the history
)
  • Loading branch information
JasonKYi committed Feb 28, 2021
1 parent 9668bdd commit 11f1801
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/linear_algebra/quadratic_form.lean
Expand Up @@ -428,6 +428,14 @@ quadratic_form.ext $ λ x,
= ⅟2 * (Q x + Q x) : by simp [map_add_self, bit0, add_mul, add_assoc]
... = Q x : by rw [← two_mul (Q x), ←mul_assoc, inv_of_mul_self, one_mul]

lemma associated_eq_self_apply (x : M) : associated Q x x = Q x :=
begin
rw [associated_apply, map_add_self],
suffices : 2 * Q x * ⅟ 2 = Q x,
{ ring, assumption },
rw [mul_right_comm, mul_inv_of_self, one_mul],
end

end associated

section anisotropic
Expand Down

0 comments on commit 11f1801

Please sign in to comment.