Documentation

Mathlib.CategoryTheory.Limits.Shapes.SequentialProduct

ℕ-indexed products as sequential limits #

Given sequences M N : ℕ → C of objects with morphisms f n : M n ⟶ N n for all n, this file exhibits ∏ M as the limit of the tower

⋯ → ∏_{n < m + 1} M n × ∏_{n ≥ m + 1} N n → ∏_{n < m} M n × ∏_{n ≥ m} N n → ⋯ → ∏ N

Further, we prove that the transition maps in this tower are epimorphisms, in the case when each f n is an epimorphism and C has finite biproducts.

theorem CategoryTheory.Limits.SequentialProduct.functorObj_eq_pos {C : Type u_1} {M N : C} {n m : } (h : m < n) :
(fun (i : ) => if x : i < n then M i else N i) m = M m
theorem CategoryTheory.Limits.SequentialProduct.functorObj_eq_neg {C : Type u_1} {M N : C} {n m : } (h : ¬m < n) :
(fun (i : ) => if x : i < n then M i else N i) m = N m

The product of the m first objects of M and the rest of the rest of N

Equations
Instances For

    The projection map from functorObj M N n to M m, when m < n

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

      The projection map from functorObj M N n to N m, when m ≥ n

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

        The transition maps in the sequential limit of products

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

          The cone over the tower

          ⋯ → ∏_{n < m} M n × ∏_{n ≥ m} N n → ⋯ → ∏ N
          

          with cone point ∏ M. This is a limit cone, see CategoryTheory.Limits.SequentialProduct.isLimit.

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

            The cone over the tower

            ⋯ → ∏_{n < m} M n × ∏_{n ≥ m} N n → ⋯ → ∏ N
            

            with cone point ∏ M is indeed a limit cone.

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