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

Commit b1c1033

Browse files
committed
feat(analysis/normed_space/operator_norm): construct a continuous_linear_equiv from a linear_equiv and bounds in both directions (#4583)
1 parent 7cff825 commit b1c1033

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

src/analysis/normed_space/operator_norm.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -900,6 +900,14 @@ continuous_linear_equiv.uniform_embedding
900900
continuous_inv_fun := h₂,
901901
.. e }
902902

903+
/-- Construct a continuous linear equivalence from a linear equivalence together with
904+
bounds in both directions. -/
905+
def linear_equiv.to_continuous_linear_equiv_of_bounds (e : E ≃ₗ[𝕜] F) (C_to C_inv : ℝ)
906+
(h_to : ∀ x, ∥e x∥ ≤ C_to * ∥x∥) (h_inv : ∀ x : F, ∥e.symm x∥ ≤ C_inv * ∥x∥) : E ≃L[𝕜] F :=
907+
{ to_linear_equiv := e,
908+
continuous_to_fun := e.to_linear_map.continuous_of_bound C_to h_to,
909+
continuous_inv_fun := e.symm.to_linear_map.continuous_of_bound C_inv h_inv }
910+
903911
namespace continuous_linear_map
904912
variables (𝕜) (𝕜' : Type*) [normed_ring 𝕜'] [normed_algebra 𝕜 𝕜']
905913

0 commit comments

Comments
 (0)