Skip to content

Commit

Permalink
feat(linear_algebra/finsupp): adjust apply lemma for `finsupp.dom_lco…
Browse files Browse the repository at this point in the history
…ngr` (#7549)

This is a split-off dependency from #7496.





Co-authored-by: Vierkantor <vierkantor@vierkantor.com>
  • Loading branch information
Vierkantor and Vierkantor committed May 11, 2021
1 parent 9191a67 commit b746e82
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 5 deletions.
2 changes: 1 addition & 1 deletion src/linear_algebra/basis.lean
Expand Up @@ -250,7 +250,7 @@ funext (b.reindex_apply e)
@[simp] lemma coe_reindex_repr : ((b.reindex e).repr x : ι' → R) = b.repr x ∘ e.symm :=
funext $ λ i',
show (finsupp.dom_lcongr e : _ ≃ₗ[R] _) (b.repr x) i' = _,
from finsupp.dom_lcongr_apply _ _ _
by simp

@[simp] lemma reindex_repr (i' : ι') : (b.reindex e).repr x i' = b.repr x (e.symm i') :=
by rw coe_reindex_repr
Expand Down
8 changes: 4 additions & 4 deletions src/linear_algebra/finsupp.lean
Expand Up @@ -550,10 +550,10 @@ protected def dom_lcongr {α₁ α₂ : Type*} (e : α₁ ≃ α₂) :
(α₁ →₀ M) ≃ₗ[R] (α₂ →₀ M) :=
(finsupp.dom_congr e : (α₁ →₀ M) ≃+ (α₂ →₀ M)).to_linear_equiv (lmap_domain M R e).map_smul

lemma dom_lcongr_apply {α₁ : Type*} {α₂ : Type*} (e : α₁ ≃ α₂) (v : α₁ →₀ M) (i : α₂) :
(finsupp.dom_lcongr e : _ ≃ₗ[R] _) v i = v (e.symm i) :=
by { conv_lhs { rw ← e.apply_symm_apply i },
exact finsupp.map_domain_apply e.injective v (e.symm i) }
@[simp]
lemma dom_lcongr_apply {α₁ : Type*} {α₂ : Type*} (e : α₁ ≃ α₂) (v : α₁ →₀ M) :
(finsupp.dom_lcongr e : _ ≃ₗ[R] _) v = finsupp.dom_congr e v :=
rfl

@[simp]
lemma dom_lcongr_refl : finsupp.dom_lcongr (equiv.refl α) = linear_equiv.refl R (α →₀ M) :=
Expand Down

0 comments on commit b746e82

Please sign in to comment.