Zulip Chat Archive

Stream: condensed mathematics

Topic: Exact functors


Adam Topaz (May 11 2022 at 14:59):

Did we ever decide (in LTE and/or mathlib) how to talk about exact functors?

Johan Commelin (May 11 2022 at 15:00):

Not really. I think the idea was to say that they preserve finite (co)limits.

Johan Commelin (May 11 2022 at 15:00):

But it hasn't been connected to exact.

Riccardo Brasca (May 11 2022 at 15:06):

We have docs#category_theory.abelian.functor.preserves_exact_of_preserves_finite_colimits_of_epi and the dual docs#category_theory.abelian.functor.preserves_exact_of_preserves_finite_limits_of_mono

Adam Topaz (May 11 2022 at 15:10):

Nice, okay that should do it.

Johan Commelin (May 11 2022 at 15:10):

@Riccardo Brasca Ooh, yes of course. Why did I forget about those!? Thanks for the pointers.

Adam Topaz (May 11 2022 at 15:10):

I started an AB4.lean file which seems to be needed:
https://github.com/leanprover-community/lean-liquid/blob/master/src/for_mathlib/ab4.lean

Adam Topaz (May 11 2022 at 15:11):

We'll probably need to show that coproduct_functor is exact given AB4.

Johan Commelin (May 11 2022 at 15:13):

Is this a missing piece for showing that Ext sends coproducts to products?

Adam Topaz (May 11 2022 at 15:14):

Yeah

Adam Topaz (May 11 2022 at 15:14):

This is what's needed to show that homology commutes with coproducts.

Adam Topaz (May 11 2022 at 15:14):

(it's not true in general!)

Adam Topaz (May 11 2022 at 15:15):

https://mathoverflow.net/a/146941

Johan Commelin (May 11 2022 at 15:29):

Ok, and so we need to show that Ab satisfies AB4

Johan Commelin (May 11 2022 at 15:29):

But we don't need it for Cond(Ab), if I understand it correctly.

Adam Topaz (May 11 2022 at 15:30):

No, I think we do need it for Cond(Ab).

Adam Topaz (May 11 2022 at 15:31):

Aren't we dealing with complexes of condensed abelian groups?

Johan Commelin (May 11 2022 at 15:32):

But to compute Ext^n(foo, bar) you only take homology of a complex of abelian groups, right?

Adam Topaz (May 11 2022 at 15:33):

Oh, I should have specified -- we need this to show that a coproduct of quasi-isos is a quasi-iso.

Adam Topaz (May 11 2022 at 15:33):

Is that true without AB4?

Adam Topaz (May 11 2022 at 15:36):

Here is the target lemma:
https://github.com/leanprover-community/lean-liquid/blob/ba6f0cadbe3a895dcbaf5a70e0b1c18a42c05ea6/src/for_mathlib/derived/ext_coproducts.lean#L239

Adam Topaz (May 11 2022 at 15:36):

(is GH down?)

Johan Commelin (May 11 2022 at 15:36):

I see. I agree that AB4 certainly helps. I don't know if it is strictly necessary, but I guess it is.

Filippo A. E. Nuccio (May 11 2022 at 17:34):

In Tohoku Grothendieck works with sheaves on Top, but there he observes that sheaves in abelian groups satisfy AB5, hence AB4. Is this not enough to deduce AB4 for Cond Ab?

Adam Topaz (May 11 2022 at 17:45):

Oh, AB4 for Cond Ab should be pretty easy to prove.

Adam Topaz (May 11 2022 at 17:45):

That's not the issue, rather the issue is whether we need to prove it :)

Filippo A. E. Nuccio (May 11 2022 at 17:46):

Ah ok, I see. It sounded strange that it might not be true...

Kevin Buzzard (May 11 2022 at 18:09):

Essentially every abelian category "extra axiom" is true for Cond Ab!

Adam Topaz (May 11 2022 at 18:12):

And even better they all follow from
https://github.com/leanprover-community/lean-liquid/blob/d3188794d3b2232ff7c68c3b5e83ef2cef10d58c/src/condensed/extr/equivalence.lean#L371

Kevin Buzzard (May 11 2022 at 18:31):

For an arbitrary category C (with finite products or whatever one needs for sheaves), one can consider C-valued sheaves on extremely disconnected sets or profinite sets or compact Hausdorff sets, with the topologies we use on these categories. Are these things all the same in this generality?

Peter Scholze (May 11 2022 at 18:32):

Only if C has all limits

Peter Scholze (May 11 2022 at 18:35):

I think in general C-sheaves on CHaus are a full subcategory of C-sheaves on ProFin are a full subcategory of C-sheaves on ExtrDisc, and the essential images are given by those sheaves where the limit that wants to define the value on some compact Hausdorff (resp. profinite) actually exists in C.

Adam Topaz (May 11 2022 at 21:53):

https://github.com/leanprover-community/lean-liquid/blob/e948977da669ce56998eaa819ed5c402c0fb7002/src/condensed/ab4.lean#L178

Kevin Buzzard (May 11 2022 at 22:41):

Good old AB4_of_preserves_colimits_of_reflects_limits_of_AB4

Adam Topaz (May 11 2022 at 22:44):

What's the stacks tag for that lemma? ;)

Kevin Buzzard (May 11 2022 at 22:56):

I wonder if the Stacks proof contains lines such as swap, { rintro i _ ⟨⟨⟨⟩⟩⟩, dsimp, simp, dsimp, simp },

Kevin Buzzard (May 11 2022 at 22:57):

This really is all about knowing the correct abstractions in category theory isn't it. Very well done.


Last updated: Dec 20 2023 at 11:08 UTC