Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
feat(linear_algebra/affine_space/affine_map): add missing simp lemma …
Browse files Browse the repository at this point in the history
…`affine_map.homothety_apply_same` (#9360)
  • Loading branch information
ocfnash committed Sep 24, 2021
1 parent 48883dc commit 0db6caf
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions src/linear_algebra/affine_space/affine_map.lean
Original file line number Diff line number Diff line change
Expand Up @@ -490,6 +490,8 @@ lemma homothety_eq_line_map (c : P1) (r : k) (p : P1) : homothety c r p = line_m
@[simp] lemma homothety_one (c : P1) : homothety c (1:k) = id k P1 :=
by { ext p, simp [homothety_apply] }

@[simp] lemma homothety_apply_same (c : P1) (r : k) : homothety c r c = c := line_map_same_apply c r

lemma homothety_mul (c : P1) (r₁ r₂ : k) :
homothety c (r₁ * r₂) = (homothety c r₁).comp (homothety c r₂) :=
by { ext p, simp [homothety_apply, mul_smul] }
Expand Down

0 comments on commit 0db6caf

Please sign in to comment.