Zulip Chat Archive

Stream: maths

Topic: pseudoelements


Johan Commelin (Apr 06 2022 at 13:45):

It seems to me that pseudoelements of an object X in an abelian category form a group. Is this true? Is it in mathlib? Can we endow homsets with an add_monoid_hom_class instance?

Is the following provable?

import category_theory.abelian.pseudoelements

open category_theory category_theory.limits
open_locale pseudoelement

 lemma pseudoelement.biprod_ext {X Y : A} (p q : (X  Y))
   (h1 : (biprod.fst : X  Y  X) p = (biprod.fst : X  Y  X) q)
   (h2 : (biprod.snd : X  Y  Y) p = (biprod.snd : X  Y  Y) q) :
   p = q :=
sorry

Johan Commelin (Apr 06 2022 at 13:48):

@Markus Himmel I guess you have thought about such issues. I read a comment that doing pullbacks is hairy...

Adam Topaz (Apr 06 2022 at 13:49):

The proper way to do what I'm guessing you want is to prove the Freyd embedding theorem.

Adam Topaz (Apr 06 2022 at 13:50):

But maybe there is a more direct way with pseudoelements.... I don't know.

Riccardo Brasca (Apr 06 2022 at 13:51):

You can often use docs#category_theory.abelian.pseudoelement.sub_of_eq_image to "mimic" the difference of two pseudoelements.

Riccardo Brasca (Apr 06 2022 at 13:52):

It was enough to prove the snake lemma, where on paper one would take the difference (at least in R-mod).

Markus Himmel (Apr 06 2022 at 13:56):

The equivalence relation on the homs with codomain P is not compatible with addition-after-taking-pullbacks, so you cannot make the pseudoelements into an abelian group.

One way to fix this is by not quotienting out the equivalence relation, but then you have to do all the bookkeeping manually. This technique is described in https://math.berkeley.edu/~gbergman/papers/unpub/elem-chase.pdf

Johan Commelin (Apr 06 2022 at 14:05):

Hmm, I will try to work out what goes wrong, because I don't see it yet.

Adam Topaz (Apr 06 2022 at 14:08):

The relation involves some epi assumptions. Does that throw a wrench in things?

Johan Commelin (Apr 06 2022 at 14:18):

I guess the problem is with negation? Becuase f(f) ⁣:XXYf \oplus (-f) \colon X \oplus X \to Y is not equivalent to the zero map?

Johan Commelin (Apr 06 2022 at 14:18):

I haven't written lean code yet, but getting a monoid seems to be ok

Adam Topaz (Apr 06 2022 at 14:19):

What about associativity of addition?

Johan Commelin (Apr 06 2022 at 14:20):

I think that should be fine, since (XY)ZX(YZ)(X \oplus Y) \oplus Z \cong X \oplus (Y \oplus Z). The problem is axioms that reduce arity. Afaict.

Adam Topaz (Apr 06 2022 at 14:21):

Yeah that's right.

Adam Topaz (Apr 06 2022 at 14:21):

You would take that isomorphism as your epi

Markus Himmel (Apr 06 2022 at 14:53):

f(f)f \oplus (-f) cannot be equivalent to the zero map unless f=0f = 0 since the only things that are equivalent to zero maps are zero maps. See docs#category_theory.abelian.pseudoelement.pseudo_zero_aux

Kevin Buzzard (Apr 06 2022 at 15:18):

Aah so maybe it's a monoid :-)

Johan Commelin (Apr 07 2022 at 06:43):

So here's a lemma that I've been trying to prove using pseudoelements, but I failed so far:
https://github.com/leanprover-community/lean-liquid/blob/master/src/for_mathlib/derived/les.lean#L128

I would be interested in seeing a proof that works. Because I think that a proof without pseudoelements will quickly be ugly.


Last updated: Dec 20 2023 at 11:08 UTC