Zulip Chat Archive

Stream: general

Topic: Translating Module.exact_iff to Ab


Fabian Glöckle (Mar 01 2022 at 12:51):

Hi, I am trying to prove the equivalent statement to docs#Module.exact_iff for AddCommGroup instead of Module, i.e.

theorem exact_iff {M N O : AddCommGroup.{v}} (f : M  N) (g : N  O): exact f g  f.range = g.ker := sorry

If you can explain me why this isn't needed or how to do it with the forgetful functor from Module \Z, I'd be very grateful.
For now, I thought I'll have to translate the proof, which involves first getting the respective statements for docs#Module.kernel_cone, docs#Module.kernel_is_limit etc.
@Markus Himmel It seems you have written this for Module. What yould you recommend?

Riccardo Brasca (Mar 01 2022 at 12:55):

I would prove that an equivalences of categories preserves exactness (that it's relevant in its own). Then I suppose we know that the forgetful functor is an equivalence. But it's very possible there is a shorter way.

Fabian Glöckle (Mar 01 2022 at 12:58):

yes, we do know that

Markus Himmel (Mar 01 2022 at 12:58):

If you know that the forgetful functor preserves and reflects exact sequences then it should be easy

Riccardo Brasca (Mar 01 2022 at 13:01):

So this is a good reason to finish my review of #12071

Fabian Glöckle (Mar 01 2022 at 13:02):

uhh, nice!

Riccardo Brasca (Mar 01 2022 at 13:09):

So I really suggest to prove the general about equivalences of categories, and use it.

Johan Commelin (Mar 01 2022 at 16:31):

@Fabian Glöckle AddCommGroup.exact_iff is already in LTE.

Fabian Glöckle (Mar 01 2022 at 16:34):

ohh

Fabian Glöckle (Mar 01 2022 at 16:35):

wait, doesn't VSCode Ctrl-T search your own src/ as well?

Johan Commelin (Mar 01 2022 at 16:36):

Je ne sais pas. But I think you want

src/for_mathlib/AddCommGroup/exact.lean
12:theorem exact_iff : exact f g  f.range = g.ker :=

Fabian Glöckle (Mar 01 2022 at 16:36):

yes yes I've found it

Fabian Glöckle (Mar 01 2022 at 16:37):

but I thought I had checked in advance what's there

Fabian Glöckle (Mar 01 2022 at 16:37):

so do you grep your repo to find lemmas others have written or do you all just have a very good overview over what's there?

Fabian Glöckle (Mar 01 2022 at 16:38):

and so you did rewrite the def kernel_is_limit : is_limit (kernel_cone f) :D

Fabian Glöckle (Mar 01 2022 at 16:38):

thank you a lot
that saved me a bunch of time!

Johan Commelin (Mar 01 2022 at 17:40):

Fabian Glöckle said:

so do you grep your repo to find lemmas others have written or do you all just have a very good overview over what's there?

both (-;

Riccardo Brasca (Mar 03 2022 at 21:27):

@Markus Himmel If you're happy with #12071 don't forget to merge it!


Last updated: Dec 20 2023 at 11:08 UTC