Skip to content

Commit

Permalink
feat(linear_algebra/affine_space/affine_equiv): lemmas about coercion…
Browse files Browse the repository at this point in the history
… to `affine_map` (#16284)

Add two more `rfl` (and `simp`) lemmas about the coercion from
`affine_equiv` to `affine_map`.  In both cases very similar lemmas are
already present (in one case a version using `to_affine_map`, in one
case a version for the coercion to a function), but apparently not
these particular ones.
  • Loading branch information
jsm28 committed Aug 29, 2022
1 parent 3e2fb4c commit 39d5a98
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/linear_algebra/affine_space/affine_equiv.lean
Expand Up @@ -86,6 +86,8 @@ rfl

@[simp] lemma linear_to_affine_map (e : P₁ ≃ᵃ[k] P₂) : e.to_affine_map.linear = e.linear := rfl

@[simp] lemma coe_linear (e : P₁ ≃ᵃ[k] P₂) : (e : P₁ →ᵃ[k] P₂).linear = e.linear := rfl

lemma to_affine_map_injective : injective (to_affine_map : (P₁ ≃ᵃ[k] P₂) → (P₁ →ᵃ[k] P₂)) :=
begin
rintros ⟨e, el, h⟩ ⟨e', el', h'⟩ H,
Expand Down Expand Up @@ -206,6 +208,10 @@ include V₂ V₃

@[simp] lemma coe_trans (e : P₁ ≃ᵃ[k] P₂) (e' : P₂ ≃ᵃ[k] P₃) : ⇑(e.trans e') = e' ∘ e := rfl

@[simp] lemma coe_trans_to_affine_map (e : P₁ ≃ᵃ[k] P₂) (e' : P₂ ≃ᵃ[k] P₃) :
(e.trans e' : P₁ →ᵃ[k] P₃) = (e' : P₂ →ᵃ[k] P₃).comp e :=
rfl

@[simp]
lemma trans_apply (e : P₁ ≃ᵃ[k] P₂) (e' : P₂ ≃ᵃ[k] P₃) (p : P₁) : e.trans e' p = e' (e p) := rfl

Expand Down

0 comments on commit 39d5a98

Please sign in to comment.