Partial functions and topological spaces #
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.
theorem
rtendsto_nhds
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
{r : Rel Y X}
{l : Filter Y}
{x : X}
:
theorem
rtendsto'_nhds
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
{r : Rel Y X}
{l : Filter Y}
{x : X}
:
theorem
ptendsto_nhds
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
{f : Y →. X}
{l : Filter Y}
{x : X}
:
theorem
ptendsto'_nhds
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
{f : Y →. X}
{l : Filter Y}
{x : X}
:
Continuity and partial functions #
def
PContinuous
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
[TopologicalSpace Y]
(f : X →. Y)
:
Continuity of a partial function
Instances For
theorem
open_dom_of_pcontinuous
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
[TopologicalSpace Y]
{f : X →. Y}
(h : PContinuous f)
:
theorem
pcontinuous_iff'
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
[TopologicalSpace Y]
{f : X →. Y}
:
theorem
continuousWithinAt_iff_ptendsto_res
{X : Type u_1}
{Y : Type u_2}
[TopologicalSpace X]
[TopologicalSpace Y]
(f : X → Y)
{x : X}
{s : Set X}
: