Documentation

Mathlib.CategoryTheory.Abelian.Pseudoelements

Pseudoelements in abelian categories #

A pseudoelement of an object X in an abelian category C is an equivalence class of arrows ending in X, where two arrows are considered equivalent if we can find two epimorphisms with a common domain making a commutative square with the two arrows. While the construction shows that pseudoelements are actually subobjects of X rather than "elements", it is possible to chase these pseudoelements through commutative diagrams in an abelian category to prove exactness properties. This is done using some "diagram-chasing metatheorems" proved in this file. In many cases, a proof in the category of abelian groups can more or less directly be converted into a proof using pseudoelements.

A classic application of pseudoelements are diagram lemmas like the four lemma or the snake lemma.

Pseudoelements are in some ways weaker than actual elements in a concrete category. The most important limitation is that there is no extensionality principle: If f g : X ⟶ Y, then ∀ x ∈ X, f x = g x does not necessarily imply that f = g (however, if f = 0 or g = 0, it does). A corollary of this is that we can not define arrows in abelian categories by dictating their action on pseudoelements. Thus, a usual style of proofs in abelian categories is this: First, we construct some morphism using universal properties, and then we use diagram chasing of pseudoelements to verify that is has some desirable property such as exactness.

It should be noted that the Freyd-Mitchell embedding theorem gives a vastly stronger notion of pseudoelement (in particular one that gives extensionality). However, this theorem is quite difficult to prove and probably out of reach for a formal proof for the time being.

Main results #

We define the type of pseudoelements of an object and, in particular, the zero pseudoelement.

We prove that every morphism maps the zero pseudoelement to the zero pseudoelement (apply_zero) and that a zero morphism maps every pseudoelement to the zero pseudoelement (zero_apply).

Here are the metatheorems we provide:

Notations #

We introduce coercions from an object of an abelian category to the set of its pseudoelements and from a morphism to the function it induces on pseudoelements.

These coercions must be explicitly enabled via local instances: attribute [local instance] objectToSort homToFun

Implementation notes #

It appears that sometimes the coercion from morphisms to functions does not work, i.e., writing g a raises a "function expected" error. This error can be fixed by writing (g : X ⟶ Y) a.

References #

This is just composition of morphisms in C. Another way to express this would be (Over.map f).obj a, but our definition has nicer definitional properties.

Equations
Instances For

    Two arrows f : X ⟶ P and g : Y ⟶ P are called pseudo-equal if there is some object R and epimorphisms p : R ⟶ X and q : R ⟶ Y such that p ≫ f = q ≫ g.

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

      Pseudoequality is transitive: Just take the pullback. The pullback morphisms will be epimorphisms since in an abelian category, pullbacks of epimorphisms are epimorphisms.

      The arrows with codomain P equipped with the equivalence relation of being pseudo-equal.

      Equations
      Instances For

        A Pseudoelement of P is just an equivalence class of arrows ending in P by being pseudo-equal.

        Equations
        Instances For

          A coercion from an object of an abelian category to its pseudoelements.

          Equations
          Instances For

            A coercion from an arrow with codomain P to its associated pseudoelement.

            Equations
            Instances For

              If two elements are pseudo-equal, then their composition with a morphism is, too.

              A coercion from morphisms to functions on pseudoelements.

              Equations
              • CategoryTheory.Abelian.Pseudoelement.homToFun = { coe := CategoryTheory.Abelian.Pseudoelement.pseudoApply }
              Instances For

                Applying a pseudoelement to a composition of morphisms is the same as composing with each morphism. Sadly, this is not a definitional equality, but at least it is true.

                In this section we prove that for every P there is an equivalence class that contains precisely all the zero morphisms ending in P and use this to define the zero pseudoelement.

                The arrows pseudo-equal to a zero morphism are precisely the zero morphisms.

                The zero pseudoelement is the class of a zero morphism.

                Equations
                Instances For
                  Equations
                  • CategoryTheory.Abelian.Pseudoelement.hasZero = { zero := CategoryTheory.Abelian.Pseudoelement.pseudoZero }
                  Equations
                  • CategoryTheory.Abelian.Pseudoelement.instInhabitedPseudoelement = { default := 0 }

                  The pseudoelement induced by an arrow is zero precisely when that arrow is zero.

                  @[simp]

                  Morphisms map the zero pseudoelement to the zero pseudoelement.

                  An extensionality lemma for being the zero arrow.

                  A morphism that only maps the zero pseudoelement to zero is a monomorphism.

                  If two pseudoelements x and y have the same image under some morphism f, then we can form their "difference" z. This pseudoelement has the properties that f z = 0 and for all morphisms g, if g y = 0 then g z = g x.

                  If f : P ⟶ R and g : Q ⟶ R are morphisms and p : P and q : Q are pseudoelements such that f p = g q, then there is some s : pullback f g such that fst s = p and snd s = q.

                  Remark: Borceux claims that s is unique, but this is false. See Counterexamples/Pseudoelement.lean for details.

                  In the category Module R, if x and y are pseudoequal, then the range of the associated morphisms is the same.