Skip to content

Commit

Permalink
doc(representation_theory/basic): add docstring to dual_tensor_hom_co…
Browse files Browse the repository at this point in the history
…mm (#18661)

add a docstring to dual_tensor_hom_comm to describe its mathematical content explicitly
  • Loading branch information
PatrickKinnear committed Mar 29, 2023
1 parent 2de9c37 commit 9cb7206
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/representation_theory/basic.lean
Expand Up @@ -378,6 +378,13 @@ def dual : representation k G (module.dual k V) :=
@[simp]
lemma dual_apply (g : G) : (dual ρV) g = module.dual.transpose (ρV g⁻¹) := rfl

/--
Given $k$-modules $V, W$, there is a homomorphism $φ : V^* ⊗ W → Hom_k(V, W)$
(implemented by `linear_algebra.contraction.dual_tensor_hom`).
Given representations of $G$ on $V$ and $W$,there are representations of $G$ on $V^* ⊗ W$ and on
$Hom_k(V, W)$.
This lemma says that $φ$ is $G$-linear.
-/
lemma dual_tensor_hom_comm (g : G) :
(dual_tensor_hom k V W) ∘ₗ (tensor_product.map (ρV.dual g) (ρW g)) =
(lin_hom ρV ρW) g ∘ₗ (dual_tensor_hom k V W) :=
Expand Down

0 comments on commit 9cb7206

Please sign in to comment.