Documentation

Mathlib.Topology.Instances.Real.Lemmas

Topological properties of ℝ #

theorem Real.isTopologicalBasis_Ioo_rat :
TopologicalSpace.IsTopologicalBasis (⋃ (a : ), ⋃ (b : ), ⋃ (_ : a < b), {Set.Ioo a b})
theorem Real.mem_closure_iff {s : Set } {x : } :
x closure s ε > 0, ys, |y - x| < ε
theorem Real.uniformContinuous_inv (s : Set ) {r : } (r0 : 0 < r) (H : xs, r |x|) :
UniformContinuous fun (p : s) => (↑p)⁻¹
theorem Real.continuous_inv :
Continuous fun (a : { r : // r 0 }) => (↑a)⁻¹
theorem Real.uniformContinuous_mul (s : Set ( × )) {r₁ r₂ : } (H : xs, |x.1| < r₁ |x.2| < r₂) :
UniformContinuous fun (p : s) => (↑p).1 * (↑p).2
theorem closure_of_rat_image_lt {q : } :
closure (Rat.cast '' {x : | q < x}) = {r : | q r}
theorem Function.Periodic.compact_of_continuous {α : Type u} [TopologicalSpace α] {f : α} {c : } (hp : Function.Periodic f c) (hc : c 0) (hf : Continuous f) :

A continuous, periodic function has compact range.

theorem Function.Periodic.isBounded_of_continuous {α : Type u} [PseudoMetricSpace α] {f : α} {c : } (hp : Function.Periodic f c) (hc : c 0) (hf : Continuous f) :

A continuous, periodic function is bounded.