Partial functions and topological spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove properties of filter.ptendsto
etc in topological spaces. We also introduce
pcontinuous
, a version of continuous
for partially defined functions.
Continuity and partial functions #
def
pcontinuous
{α : Type u_1}
{β : Type u_2}
[topological_space α]
[topological_space β]
(f : α →. β) :
Prop
Continuity of a partial function
theorem
open_dom_of_pcontinuous
{α : Type u_1}
{β : Type u_2}
[topological_space α]
[topological_space β]
{f : α →. β}
(h : pcontinuous f) :
theorem
pcontinuous_iff'
{α : Type u_1}
{β : Type u_2}
[topological_space α]
[topological_space β]
{f : α →. β} :
pcontinuous f ↔ ∀ {x : α} {y : β}, y ∈ f x → filter.ptendsto' f (nhds x) (nhds y)
theorem
continuous_within_at_iff_ptendsto_res
{α : Type u_1}
{β : Type u_2}
[topological_space α]
[topological_space β]
(f : α → β)
{x : α}
{s : set α} :
continuous_within_at f s x ↔ filter.ptendsto (pfun.res f s) (nhds x) (nhds (f x))