Skip to content

Commit

Permalink
chore(analysis/normed_space/pi_Lp): add `pi_Lp.continuous_linear_equi…
Browse files Browse the repository at this point in the history
…v` (#19014)

This bundling is often useful to have.
We keep around `pi_Lp.linear_equiv` as this is shorter to write than `pi_Lp.continuous_linear_equiv.to_linear_equiv`.
  • Loading branch information
eric-wieser committed May 15, 2023
1 parent 4b884ef commit e9f2a83
Showing 1 changed file with 8 additions and 1 deletion.
9 changes: 8 additions & 1 deletion src/analysis/normed_space/pi_Lp.lean
Expand Up @@ -707,13 +707,20 @@ lemma norm_equiv_symm_one {β} [seminormed_add_comm_group β] (hp : p ≠ ∞) [

variables (𝕜 p)

/-- `pi_Lp.equiv` as a linear map. -/
/-- `pi_Lp.equiv` as a linear equivalence. -/
@[simps {fully_applied := ff}]
protected def linear_equiv : pi_Lp p β ≃ₗ[𝕜] Π i, β i :=
{ to_fun := pi_Lp.equiv _ _,
inv_fun := (pi_Lp.equiv _ _).symm,
..linear_equiv.refl _ _}

/-- `pi_Lp.equiv` as a continuous linear equivalence. -/
@[simps {fully_applied := ff}]
protected def continuous_linear_equiv : pi_Lp p β ≃L[𝕜] Π i, β i :=
{ to_linear_equiv := pi_Lp.linear_equiv _ _ _,
continuous_to_fun := continuous_equiv _ _,
continuous_inv_fun := continuous_equiv_symm _ _ }

section basis

variables (ι)
Expand Down

0 comments on commit e9f2a83

Please sign in to comment.