Pseudoelements and pullbacks #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4. Borceux claims in Proposition 1.9.5 that the pseudoelement constructed in
category_theory.abelian.pseudoelement.pseudo_pullback
is unique. We show here that this claim is false. This means in particular that we cannot have an extensionality principle for pullbacks in terms of pseudoelements.
Implementation details #
The construction, suggested in https://mathoverflow.net/a/419951/7845, is the following.
We work in the category of Module ℤ
and we consider the special case of ℚ ⊞ ℚ
(that is the
pullback over the terminal object). We consider the pseudoelements associated to x : ℚ ⟶ ℚ ⊞ ℚ
given by t ↦ (t, 2 * t)
and y : ℚ ⟶ ℚ ⊞ ℚ
given by t ↦ (t, t)
.
Main results #
category_theory.abelian.pseudoelement.exist_ne_and_fst_eq_fst_and_snd_eq_snd
: there are two pseudoelementsx y : ℚ ⊞ ℚ
such thatx ≠ y
,biprod.fst x = biprod.fst y
andbiprod.snd x = biprod.snd y
.
References #
x
is given by t ↦ (t, 2 * t)
.
y
is given by t ↦ (t, t)
.
biprod.fst ≫ x
is pseudoequal to biprod.fst y
.
biprod.snd ≫ x
is pseudoequal to biprod.snd y
.
x
is not pseudoequal to y
.
biprod.fst ⟦x⟧ = biprod.fst ⟦y⟧
.
biprod.snd ⟦x⟧ = biprod.snd ⟦y⟧
.
There are two pseudoelements x y : ℚ ⊞ ℚ
such that x ≠ y
, biprod.fst x = biprod.fst y
and
biprod.snd x = biprod.snd y
.