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_pt (R A B : Type u) [CommRing R] [CommRing A] [CommRing B] [Algebra R A] [Algebra R B] :
    (pushoutCocone R A B).pt = { carrier := TensorProduct R A B, commRing := Algebra.TensorProduct.instCommRing }

    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_iff_isPushout {R S : Type u} [CommRing R] [CommRing S] [Algebra R S] {R' S' : Type u} [CommRing R'] [CommRing S'] [Algebra R R'] [Algebra S S'] [Algebra R' S'] [Algebra R S'] [IsScalarTower R R' S'] [IsScalarTower R S S'] :

      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

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

        Equations
        Instances For
          Equations

          The trivial ring is the (strict) terminal object of CommRingCat.

          Equations
          Instances For

            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 = { carrier := A × B, commRing := Prod.instCommRing }

              The product in CommRingCat is the Cartesian product.

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

                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) :
                  (piFan R).pt = { carrier := (i : ι) → (R i), commRing := Pi.commRing }

                  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 { carrier := (i : ι) → (R i), commRing := Pi.commRing }

                    The categorical product and the usual product agree

                    Equations
                    Instances For
                      noncomputable def RingEquiv.piEquivPi {ι : Type u} (R : ιType u) [(i : ι) → CommRing (R i)] :
                      ↑(∏ᶜ fun (i : ι) => { carrier := R i, commRing := inst✝ i }) ≃+* ((i : ι) → R i)

                      The categorical product and the usual product agree

                      Equations
                      Instances For

                        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

                            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