Documentation

Mathlib.Topology.MetricSpace.Pseudo.Lemmas

Extra lemmas about pseudo-metric spaces #

theorem Real.singleton_eq_inter_Icc (b : ) :
{b} = ⋂ (r : ), ⋂ (_ : r > 0), Set.Icc (b - r) (b + r)
theorem squeeze_zero' {α : Type u_3} {f : α} {g : α} {t₀ : Filter α} (hf : ∀ᶠ (t : α) in t₀, 0 f t) (hft : ∀ᶠ (t : α) in t₀, f t g t) (g0 : Filter.Tendsto g t₀ (nhds 0)) :
Filter.Tendsto f t₀ (nhds 0)

Special case of the sandwich lemma; see tendsto_of_tendsto_of_tendsto_of_le_of_le' for the general case.

theorem squeeze_zero {α : Type u_3} {f : α} {g : α} {t₀ : Filter α} (hf : ∀ (t : α), 0 f t) (hft : ∀ (t : α), f t g t) (g0 : Filter.Tendsto g t₀ (nhds 0)) :
Filter.Tendsto f t₀ (nhds 0)

Special case of the sandwich lemma; see tendsto_of_tendsto_of_tendsto_of_le_of_le and tendsto_of_tendsto_of_tendsto_of_le_of_le' for the general case.

theorem eventually_closedBall_subset {α : Type u_2} [PseudoMetricSpace α] {x : α} {u : Set α} (hu : u nhds x) :
∀ᶠ (r : ) in nhds 0, Metric.closedBall x r u

If u is a neighborhood of x, then for small enough r, the closed ball Metric.closedBall x r is contained in u.

theorem Metric.isClosed_ball {α : Type u_2} [PseudoMetricSpace α] {x : α} {ε : } :
theorem Metric.isClosed_sphere {α : Type u_2} [PseudoMetricSpace α] {x : α} {ε : } :
@[simp]
@[simp]
theorem Metric.closure_sphere {α : Type u_2} [PseudoMetricSpace α] {x : α} {ε : } :