Documentation

Mathlib.Algebra.Category.Ring.Constructions

Constructions of (co)limits in CommRingCat #

In this file we provide the explicit (co)cones for various (co)limits in CommRingCat, including

The explicit cocone with tensor products as the fibered product in CommRingCat.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CommRingCat.pushoutCocone_inl (R A B : Type u) [CommRing R] [CommRing A] [CommRing B] [Algebra R A] [Algebra R B] :
    (CommRingCat.pushoutCocone R A B).inl = CommRingCat.ofHom Algebra.TensorProduct.includeLeftRingHom
    @[simp]
    theorem CommRingCat.pushoutCocone_inr (R A B : Type u) [CommRing R] [CommRing A] [CommRing B] [Algebra R A] [Algebra R B] :
    (CommRingCat.pushoutCocone R A B).inr = CommRingCat.ofHom Algebra.TensorProduct.includeRight.toRingHom

    Verify that the pushout_cocone is indeed the colimit.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem CommRingCat.isPushout_tensorProduct (R A B : Type u) [CommRing R] [CommRing A] [CommRing B] [Algebra R A] [Algebra R B] :
      CategoryTheory.IsPushout (CommRingCat.ofHom (algebraMap R A)) (CommRingCat.ofHom (algebraMap R B)) (CommRingCat.ofHom Algebra.TensorProduct.includeLeftRingHom) (CommRingCat.ofHom Algebra.TensorProduct.includeRight.toRingHom)

      The tensor product A ⊗[ℤ] B forms a cocone for A and B.

      Equations
      Instances For
        @[simp]
        theorem CommRingCat.coproductCocone_ι (A B : CommRingCat) :
        (A.coproductCocone B) = { app := fun (x : CategoryTheory.Discrete CategoryTheory.Limits.WalkingPair) => match x.as with | CategoryTheory.Limits.WalkingPair.left => CommRingCat.ofHom Algebra.TensorProduct.includeLeft | CategoryTheory.Limits.WalkingPair.right => CommRingCat.ofHom Algebra.TensorProduct.includeRight, naturality := }
        @[simp]
        theorem CommRingCat.coproductCocone_pt (A B : CommRingCat) :
        (A.coproductCocone B).pt = CommRingCat.of (TensorProduct A B)
        @[simp]
        theorem CommRingCat.coproductCocone_inl (A B : CommRingCat) :
        (A.coproductCocone B).inl = CommRingCat.ofHom Algebra.TensorProduct.includeLeft.toRingHom
        @[simp]
        theorem CommRingCat.coproductCocone_inr (A B : CommRingCat) :
        (A.coproductCocone B).inr = CommRingCat.ofHom Algebra.TensorProduct.includeRight.toRingHom

        The tensor product A ⊗[ℤ] B is a coproduct for A and B.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem CommRingCat.coproductCoconeIsColimit_desc_hom (A B : CommRingCat) (s : CategoryTheory.Limits.BinaryCofan A B) :
          ((A.coproductCoconeIsColimit B).desc s).hom = (Algebra.TensorProduct.lift s.inl.hom.toIntAlgHom s.inr.hom.toIntAlgHom ).toRingHom

          The limit cone of the tensor product A ⊗[ℤ] B in CommRingCat.

          Equations
          • A.coproductColimitCocone B = { cocone := A.coproductCocone B, isColimit := A.coproductCoconeIsColimit B }
          Instances For
            Equations
            • X.instUniqueHomOfPUnit = { default := CommRingCat.ofHom { toMonoidHom := 1, map_zero' := , map_add' := }, uniq := }

            The product in CommRingCat is the cartesian product. This is the binary fan.

            Equations
            Instances For
              @[simp]
              theorem CommRingCat.prodFan_pt (A B : CommRingCat) :
              (A.prodFan B).pt = CommRingCat.of (A × B)

              The product in CommRingCat is the cartesian product.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                noncomputable def CommRingCat.piFan {ι : Type u} (R : ιCommRingCat) :

                The categorical product of rings is the cartesian product of rings. This is its Fan.

                Equations
                Instances For
                  @[simp]
                  theorem CommRingCat.piFan_pt {ι : Type u} (R : ιCommRingCat) :
                  (CommRingCat.piFan R).pt = CommRingCat.of ((i : ι) → (R i))

                  The categorical product of rings is the cartesian product of rings.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    noncomputable def CommRingCat.piIsoPi {ι : Type u} (R : ιCommRingCat) :
                    ∏ᶜ R CommRingCat.of ((i : ι) → (R i))

                    The categorical product and the usual product agrees

                    Equations
                    Instances For
                      noncomputable def RingEquiv.piEquivPi {ι : Type u} (R : ιType u) [(i : ι) → CommRing (R i)] :
                      (∏ᶜ fun (i : ι) => CommRingCat.of (R i)) ≃+* ((i : ι) → R i)

                      The categorical product and the usual product agrees

                      Equations
                      Instances For
                        noncomputable def CommRingCat.equalizerFork {A B : CommRingCat} (f g : A B) :

                        The equalizer in CommRingCat is the equalizer as sets. This is the equalizer fork.

                        Equations
                        Instances For

                          The equalizer in CommRingCat is the equalizer as sets.

                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            noncomputable def CommRingCat.pullbackCone {A B C : CommRingCat} (f : A C) (g : B C) :

                            In the category of CommRingCat, the pullback of f : A ⟶ C and g : B ⟶ C is the eqLocus of the two maps A × B ⟶ C. This is the constructed pullback cone.

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

                              The constructed pullback cone is indeed the limit.

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