Documentation

Mathlib.CategoryTheory.Category.PartialFun

The category of types with partial functions #

This defines PartialFun, the category of types equipped with partial functions.

This category is classically equivalent to the category of pointed types. The reason it doesn't hold constructively stems from the difference between Part and Option. Both can model partial functions, but the latter forces a decidable domain.

Precisely, PartialFunToPointed turns a partial function α →. β into a function Option α → Option β by sending to none the undefined values (and none to none). But being defined is (generally) undecidable while being sent to none is decidable. So it can't be constructive.

References #

def PartialFun :
Type (u_3 + 1)

The category of types equipped with partial functions.

Equations
Instances For

    Turns a type into a PartialFun.

    Equations
    Instances For
      @[simp]
      theorem PartialFun.Iso.mk_hom {α : PartialFun} {β : PartialFun} (e : α β) (x : α) :
      (PartialFun.Iso.mk e).hom x = (some (e x))
      @[simp]
      theorem PartialFun.Iso.mk_inv {α : PartialFun} {β : PartialFun} (e : α β) (x : β) :
      (PartialFun.Iso.mk e).inv x = (some (e.symm x))
      def PartialFun.Iso.mk {α : PartialFun} {β : PartialFun} (e : α β) :
      α β

      Constructs a partial function isomorphism between types from an equivalence between them.

      Equations
      • PartialFun.Iso.mk e = { hom := fun (x : α) => (some (e x)), inv := fun (x : β) => (some (e.symm x)), hom_inv_id := , inv_hom_id := }
      Instances For

        The forgetful functor from Type to PartialFun which forgets that the maps are total.

        Equations
        Instances For
          @[simp]
          theorem pointedToPartialFun_obj (X : Pointed) :
          pointedToPartialFun.obj X = { x : X.X // x X.point }
          @[simp]
          theorem pointedToPartialFun_map :
          ∀ {X Y : Pointed} (f : X Y) (a : { x : X.X // x X.point }), pointedToPartialFun.map f a = (PFun.toSubtype (fun (x : Y.X) => x Y.point) f.toFun Subtype.val) a

          The functor which deletes the point of a pointed type. In return, this makes the maps partial. This is the computable part of the equivalence PartialFunEquivPointed.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem partialFunToPointed_map :
            ∀ {X Y : PartialFun} (f : X Y), partialFunToPointed.map f = { toFun := Option.elim' none fun (a : X) => Part.toOption (f a), map_point := }
            @[simp]
            theorem partialFunToPointed_obj (X : PartialFun) :
            partialFunToPointed.obj X = { X := Option X, point := none }

            The functor which maps undefined values to a new point. This makes the maps total and creates pointed types. This is the noncomputable part of the equivalence PartialFunEquivPointed. It can't be computable because = Option.none is decidable while the domain of a general Part isn't.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              theorem partialFunEquivPointed_unitIso_hom_app (X : PartialFun) :
              partialFunEquivPointed.unitIso.hom.app X = CategoryTheory.CategoryStruct.comp (PartialFun.Iso.mk { toFun := fun (a : X) => { val := some a, property := }, invFun := fun (a : { x : Option X // ¬x = none }) => Option.get a , left_inv := , right_inv := }).hom (CategoryTheory.CategoryStruct.comp (pointedToPartialFun.map (Pointed.Iso.mk (Equiv.optionSubtypeNe none) ).inv) (pointedToPartialFun.map { toFun := Option.elim' none fun (a : { x : Option X // ¬x = none }) => a, map_point := }))
              @[simp]
              @[simp]
              theorem partialFunEquivPointed_inverse_map_get_coe :
              ∀ {X Y : Pointed} (f : X Y) (a : { x : X.X // x X.point }) (property : f.toFun a Y.point), ((partialFunEquivPointed.inverse.map f a).get property) = f.toFun a
              @[simp]
              theorem partialFunEquivPointed_inverse_obj (X : Pointed) :
              partialFunEquivPointed.inverse.obj X = { x : X.X // ¬x = X.point }
              @[simp]
              theorem partialFunEquivPointed_unitIso_inv_app (X : PartialFun) :
              partialFunEquivPointed.unitIso.inv.app X = CategoryTheory.CategoryStruct.comp (pointedToPartialFun.map { toFun := Option.elim' none fun (a : X) => some { val := some a, property := }, map_point := }) (CategoryTheory.CategoryStruct.comp (pointedToPartialFun.map (Pointed.Iso.mk (Equiv.optionSubtypeNe none) ).hom) (PartialFun.Iso.mk { toFun := fun (a : X) => { val := some a, property := }, invFun := fun (a : { x : Option X // ¬x = none }) => Option.get a , left_inv := , right_inv := }).inv)
              @[simp]
              theorem partialFunEquivPointed_functor_map_toFun :
              ∀ {X Y : PartialFun} (f : X Y) (a : Option X), (partialFunEquivPointed.functor.map f).toFun a = Option.elim' none (fun (a : X) => Part.toOption (f a)) a
              @[simp]
              theorem partialFunEquivPointed_inverse_map_Dom :
              ∀ {X Y : Pointed} (f : X Y) (a : { x : X.X // x X.point }), (partialFunEquivPointed.inverse.map f a).Dom = ¬f.toFun a = Y.point
              @[simp]
              theorem partialFunEquivPointed_counitIso_inv_app_toFun (X : Pointed) (a : ((CategoryTheory.Functor.id Pointed).obj X).X) :
              (partialFunEquivPointed.counitIso.inv.app X).toFun a = if h : a = X.point then none else some { val := a, property := h }

              The equivalence induced by PartialFunToPointed and PointedToPartialFun. Part.equivOption made functorial.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                Forgetting that maps are total and making them total again by adding a point is the same as just adding a point.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For