Skip to content

Commit 349b843

Browse files
committed
feat(Normed/Group): add lt version of IsBounded.exists_pos_norm_le (#10861)
1 parent d76a6b4 commit 349b843

File tree

2 files changed

+6
-2
lines changed

2 files changed

+6
-2
lines changed

Mathlib/Analysis/Normed/Group/Basic.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -767,6 +767,11 @@ theorem Bornology.IsBounded.exists_pos_norm_le' (hs : IsBounded s) : ∃ R > 0,
767767
#align metric.bounded.exists_pos_norm_le' Bornology.IsBounded.exists_pos_norm_le'
768768
#align metric.bounded.exists_pos_norm_le Bornology.IsBounded.exists_pos_norm_le
769769

770+
@[to_additive Bornology.IsBounded.exists_pos_norm_lt]
771+
theorem Bornology.IsBounded.exists_pos_norm_lt' (hs : IsBounded s) : ∃ R > 0, ∀ x ∈ s, ‖x‖ < R :=
772+
let ⟨R, hR₀, hR⟩ := hs.exists_pos_norm_le'
773+
⟨R + 1, by positivity, fun x hx ↦ (hR x hx).trans_lt (lt_add_one _)⟩
774+
770775
@[to_additive (attr := simp 1001) mem_sphere_iff_norm]
771776
-- Porting note: increase priority so the left-hand side doesn't reduce
772777
theorem mem_sphere_iff_norm' : b ∈ sphere a r ↔ ‖b / a‖ = r := by simp [dist_eq_norm_div]

Mathlib/Analysis/NormedSpace/lpSpace.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1174,8 +1174,7 @@ theorem norm_le_of_tendsto {C : ℝ} {F : ι → lp E p} (hCF : ∀ᶠ k in l,
11741174
/-- If `f` is the pointwise limit of a bounded sequence in `lp E p`, then `f` is in `lp E p`. -/
11751175
theorem memℓp_of_tendsto {F : ι → lp E p} (hF : Bornology.IsBounded (Set.range F)) {f : ∀ a, E a}
11761176
(hf : Tendsto (id fun i => F i : ι → ∀ a, E a) l (𝓝 f)) : Memℓp f p := by
1177-
obtain ⟨C, _, hCF'⟩ := hF.exists_pos_norm_le
1178-
have hCF : ∀ k, ‖F k‖ ≤ C := fun k => hCF' _ ⟨k, rfl⟩
1177+
obtain ⟨C, hCF⟩ : ∃ C, ∀ k, ‖F k‖ ≤ C := hF.exists_norm_le.imp fun _ ↦ Set.forall_mem_range.1
11791178
rcases eq_top_or_lt_top p with (rfl | hp)
11801179
· apply memℓp_infty
11811180
use C

0 commit comments

Comments
 (0)