Documentation

Mathlib.Topology.Order.Hom.Basic

Continuous order homomorphisms #

This file defines continuous order homomorphisms, that is maps which are both continuous and monotone. They are also called Priestley homomorphisms because they are the morphisms of the category of Priestley spaces.

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 ContinuousOrderHom (α : Type u_6) (β : Type u_7) [Preorder α] [Preorder β] [TopologicalSpace α] [TopologicalSpace β] extends OrderHom :
Type (max u_6 u_7)

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

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

    ContinuousOrderHomClass F α β states that F is a type of continuous monotone maps.

    You should extend this class when you extend ContinuousOrderHom.

    Instances
      instance ContinuousOrderHomClass.toOrderHomClass {F : Type u_1} {α : Type u_2} {β : Type u_3} [Preorder α] [Preorder β] [TopologicalSpace α] [TopologicalSpace β] [FunLike F α β] [ContinuousOrderHomClass F α β] :
      Equations
      • =
      def ContinuousOrderHomClass.toContinuousOrderHom {F : Type u_1} {α : Type u_2} {β : Type u_3} [Preorder α] [Preorder β] [TopologicalSpace α] [TopologicalSpace β] [FunLike F α β] [ContinuousOrderHomClass F α β] (f : F) :
      α →Co β

      Turn an element of a type F satisfying ContinuousOrderHomClass F α β into an actual ContinuousOrderHom. This is declared as the default coercion from F to α →Co β.

      Equations
      • f = { toOrderHom := { toFun := f, monotone' := }, continuous_toFun := }
      Instances For
        instance ContinuousOrderHomClass.instCoeTCContinuousOrderHom {F : Type u_1} {α : Type u_2} {β : Type u_3} [Preorder α] [Preorder β] [TopologicalSpace α] [TopologicalSpace β] [FunLike F α β] [ContinuousOrderHomClass F α β] :
        CoeTC F (α →Co β)
        Equations
        • ContinuousOrderHomClass.instCoeTCContinuousOrderHom = { coe := ContinuousOrderHomClass.toContinuousOrderHom }

        Top homomorphisms #

        def ContinuousOrderHom.toContinuousMap {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] (f : α →Co β) :
        C(α, β)

        Reinterpret a ContinuousOrderHom as a ContinuousMap.

        Equations
        Instances For
          instance ContinuousOrderHom.instFunLike {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] :
          FunLike (α →Co β) α β
          Equations
          • ContinuousOrderHom.instFunLike = { coe := fun (f : α →Co β) => f.toFun, coe_injective' := }
          @[simp]
          theorem ContinuousOrderHom.coe_toOrderHom {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] (f : α →Co β) :
          f.toOrderHom = f
          theorem ContinuousOrderHom.toFun_eq_coe {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] {f : α →Co β} :
          f.toFun = f
          theorem ContinuousOrderHom.ext {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] {f : α →Co β} {g : α →Co β} (h : ∀ (a : α), f a = g a) :
          f = g
          def ContinuousOrderHom.copy {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] (f : α →Co β) (f' : αβ) (h : f' = f) :
          α →Co β

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

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

            id as a ContinuousOrderHom.

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

              Composition of ContinuousOrderHoms as a ContinuousOrderHom.

              Equations
              Instances For
                @[simp]
                theorem ContinuousOrderHom.coe_comp {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] [TopologicalSpace γ] [Preorder γ] (f : β →Co γ) (g : α →Co β) :
                (ContinuousOrderHom.comp f g) = f g
                @[simp]
                theorem ContinuousOrderHom.comp_apply {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] [TopologicalSpace γ] [Preorder γ] (f : β →Co γ) (g : α →Co β) (a : α) :
                (ContinuousOrderHom.comp f g) a = f (g a)
                @[simp]
                @[simp]
                theorem ContinuousOrderHom.cancel_right {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] [TopologicalSpace γ] [Preorder γ] {g₁ : β →Co γ} {g₂ : β →Co γ} {f : α →Co β} (hf : Function.Surjective f) :
                @[simp]
                theorem ContinuousOrderHom.cancel_left {α : Type u_2} {β : Type u_3} {γ : Type u_4} [TopologicalSpace α] [Preorder α] [TopologicalSpace β] [Preorder β] [TopologicalSpace γ] [Preorder γ] {g : β →Co γ} {f₁ : α →Co β} {f₂ : α →Co β} (hg : Function.Injective g) :
                Equations
                • ContinuousOrderHom.instPreorderContinuousOrderHom = Preorder.lift DFunLike.coe
                Equations
                • ContinuousOrderHom.instPartialOrderContinuousOrderHomToPreorder = PartialOrder.lift DFunLike.coe