Documentation

Mathlib.Topology.Hom.Open

Continuous open maps #

This file defines bundled continuous open maps.

We use the DFunLike design, so each type of morphisms has a companion typeclass which is meant to be satisfied by itself and all stricter types.

Types of morphisms #

Typeclasses #

structure ContinuousOpenMap (α : Type u_6) (β : Type u_7) [TopologicalSpace α] [TopologicalSpace β] extends ContinuousMap :
Type (max u_6 u_7)

The type of continuous open maps from α to β, aka Priestley homomorphisms.

Instances For
    class ContinuousOpenMapClass (F : Type u_6) (α : outParam (Type u_7)) (β : outParam (Type u_8)) [TopologicalSpace α] [TopologicalSpace β] [FunLike F α β] extends ContinuousMapClass :

    ContinuousOpenMapClass F α β states that F is a type of continuous open maps.

    You should extend this class when you extend ContinuousOpenMap.

    Instances
      instance instCoeTCContinuousOpenMap {F : Type u_1} {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] [FunLike F α β] [ContinuousOpenMapClass F α β] :
      CoeTC F (α →CO β)
      Equations
      • instCoeTCContinuousOpenMap = { coe := fun (f : F) => { toContinuousMap := f, map_open' := } }

      Continuous open maps #

      instance ContinuousOpenMap.instFunLike {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] :
      FunLike (α →CO β) α β
      Equations
      • ContinuousOpenMap.instFunLike = { coe := fun (f : α →CO β) => f.toFun, coe_injective' := }
      theorem ContinuousOpenMap.toFun_eq_coe {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] {f : α →CO β} :
      f.toFun = f
      @[simp]
      theorem ContinuousOpenMap.coe_toContinuousMap {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] (f : α →CO β) :
      f.toContinuousMap = f
      theorem ContinuousOpenMap.ext {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] {f : α →CO β} {g : α →CO β} (h : ∀ (a : α), f a = g a) :
      f = g
      def ContinuousOpenMap.copy {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] (f : α →CO β) (f' : αβ) (h : f' = f) :
      α →CO β

      Copy of a ContinuousOpenMap with a new ContinuousMap equal to the old one. Useful to fix definitional equalities.

      Equations
      Instances For
        @[simp]
        theorem ContinuousOpenMap.coe_copy {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] (f : α →CO β) (f' : αβ) (h : f' = f) :
        (ContinuousOpenMap.copy f f' h) = f'
        theorem ContinuousOpenMap.copy_eq {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [TopologicalSpace β] (f : α →CO β) (f' : αβ) (h : f' = f) :
        def ContinuousOpenMap.id (α : Type u_2) [TopologicalSpace α] :
        α →CO α

        id as a ContinuousOpenMap.

        Equations
        Instances For
          @[simp]
          @[simp]
          theorem ContinuousOpenMap.id_apply {α : Type u_2} [TopologicalSpace α] (a : α) :
          def ContinuousOpenMap.comp {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [TopologicalSpace β] [TopologicalSpace γ] (f : β →CO γ) (g : α →CO β) :
          α →CO γ

          Composition of ContinuousOpenMaps as a ContinuousOpenMap.

          Equations
          Instances For
            @[simp]
            theorem ContinuousOpenMap.coe_comp {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [TopologicalSpace β] [TopologicalSpace γ] (f : β →CO γ) (g : α →CO β) :
            (ContinuousOpenMap.comp f g) = f g
            @[simp]
            theorem ContinuousOpenMap.comp_apply {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [TopologicalSpace β] [TopologicalSpace γ] (f : β →CO γ) (g : α →CO β) (a : α) :
            (ContinuousOpenMap.comp f g) a = f (g a)
            @[simp]
            @[simp]
            theorem ContinuousOpenMap.cancel_right {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [TopologicalSpace β] [TopologicalSpace γ] {g₁ : β →CO γ} {g₂ : β →CO γ} {f : α →CO β} (hf : Function.Surjective f) :
            @[simp]
            theorem ContinuousOpenMap.cancel_left {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [TopologicalSpace β] [TopologicalSpace γ] {g : β →CO γ} {f₁ : α →CO β} {f₂ : α →CO β} (hg : Function.Injective g) :