Documentation

Mathlib.Topology.IsLocallyHomeomorph

Local homeomorphisms #

This file defines local homeomorphisms.

Main definitions #

def IsLocallyHomeomorphOn {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] (f : XY) (s : Set X) :

A function f : X → Y satisfies IsLocallyHomeomorphOn f s if each x ∈ s is contained in the source of some e : LocalHomeomorph X Y with f = e.

Instances For
    theorem IsLocallyHomeomorphOn.mk {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] (f : XY) (s : Set X) (h : ∀ (x : X), x se, x e.source ∀ (y : X), y e.sourcef y = e y) :

    Proves that f satisfies IsLocallyHomeomorphOn f s. The condition h is weaker than the definition of IsLocallyHomeomorphOn f s, since it only requires e : LocalHomeomorph X Y to agree with f on its source e.source, as opposed to on the whole space X.

    theorem IsLocallyHomeomorphOn.map_nhds_eq {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} {s : Set X} (hf : IsLocallyHomeomorphOn f s) {x : X} (hx : x s) :
    Filter.map f (nhds x) = nhds (f x)
    theorem IsLocallyHomeomorphOn.continuousAt {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} {s : Set X} (hf : IsLocallyHomeomorphOn f s) {x : X} (hx : x s) :
    theorem IsLocallyHomeomorphOn.continuousOn {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} {s : Set X} (hf : IsLocallyHomeomorphOn f s) :
    theorem IsLocallyHomeomorphOn.comp {X : Type u_1} {Y : Type u_2} {Z : Type u_3} [TopologicalSpace X] [TopologicalSpace Y] [TopologicalSpace Z] {g : YZ} {f : XY} {s : Set X} {t : Set Y} (hg : IsLocallyHomeomorphOn g t) (hf : IsLocallyHomeomorphOn f s) (h : Set.MapsTo f s t) :
    def IsLocallyHomeomorph {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] (f : XY) :

    A function f : X → Y satisfies IsLocallyHomeomorph f if each x : x is contained in the source of some e : LocalHomeomorph X Y with f = e.

    Instances For
      theorem IsLocallyHomeomorph.mk {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] (f : XY) (h : ∀ (x : X), e, x e.source ∀ (y : X), y e.sourcef y = e y) :

      Proves that f satisfies IsLocallyHomeomorph f. The condition h is weaker than the definition of IsLocallyHomeomorph f, since it only requires e : LocalHomeomorph X Y to agree with f on its source e.source, as opposed to on the whole space X.

      theorem IsLocallyHomeomorph.map_nhds_eq {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} (hf : IsLocallyHomeomorph f) (x : X) :
      Filter.map f (nhds x) = nhds (f x)
      theorem IsLocallyHomeomorph.comp {X : Type u_1} {Y : Type u_2} {Z : Type u_3} [TopologicalSpace X] [TopologicalSpace Y] [TopologicalSpace Z] {g : YZ} {f : XY} (hg : IsLocallyHomeomorph g) (hf : IsLocallyHomeomorph f) :