Documentation

Mathlib.Topology.FiberPartition

This file provides some API surrounding Function.Fiber (see Mathlib.Logic.Function.FiberPartition) in the presence of a topology on the domain of the function.

Note: this API is designed to be useful when defining the counit of the adjunction between the functor which takes a set to the condensed set corresponding to locally constant maps to that set, and the forgetful functor from the category of condensed sets to the category of sets (see PR https://github.com/leanprover-community/mathlib4/pull/14027).

def TopologicalSpace.Fiber.sigmaIsoHom {S : Type u_1} {Y : Type u_2} (f : SY) [TopologicalSpace S] :
C((x : Function.Fiber f) × x, S)

The canonical map from the disjoint union induced by f to S.

Equations
Instances For
    @[simp]
    theorem TopologicalSpace.Fiber.sigmaIsoHom_apply {S : Type u_1} {Y : Type u_2} (f : SY) [TopologicalSpace S] (x✝ : (x : Function.Fiber f) × x) :
    (TopologicalSpace.Fiber.sigmaIsoHom f) x✝ = match x✝ with | a, x => x
    def TopologicalSpace.Fiber.sigmaIncl {S : Type u_1} {Y : Type u_2} (f : SY) [TopologicalSpace S] (a : Function.Fiber f) :
    C(a, S)

    The inclusion map from a component of the disjoint union induced by f into S.

    Equations
    Instances For
      def TopologicalSpace.Fiber.sigmaInclIncl {S : Type u_1} {Y : Type u_2} (f : SY) [TopologicalSpace S] {X : Type u_3} (g : YX) (a : Function.Fiber (g f)) (b : Function.Fiber (f (TopologicalSpace.Fiber.sigmaIncl (g f) a))) :

      The inclusion map from a fiber of a composition into the intermediate fiber.

      Equations
      Instances For