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

Commit e46daa0

Browse files
committed
feat(analysis/normed_space/operator_norm): remove to_span_singleton_norm (#16654)
Remove `continuous_linear_map.to_span_singleton_norm`. It is a duplicate of `continuous_linear_map.norm_to_span_singleton` (which has more explicit arguments and weaker type-class assumptions).
1 parent 1a4f927 commit e46daa0

File tree

1 file changed

+0
-3
lines changed

1 file changed

+0
-3
lines changed

src/analysis/normed_space/operator_norm.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1258,9 +1258,6 @@ begin
12581258
simpa only [hf, hx, mul_le_mul_right] using f.le_op_norm x,
12591259
end
12601260

1261-
lemma to_span_singleton_norm (x : E) : ∥to_span_singleton 𝕜 x∥ = ∥x∥ :=
1262-
homothety_norm _ (to_span_singleton_homothety 𝕜 x)
1263-
12641261
variable (f)
12651262

12661263
theorem uniform_embedding_of_bound {K : ℝ≥0} (hf : ∀ x, ∥x∥ ≤ K * ∥f x∥) :

0 commit comments

Comments
 (0)