Zulip Chat Archive
Stream: condensed mathematics
Topic: computing Ext with acyclics
Johan Commelin (May 19 2022 at 14:50):
I basically have the following sorry-free
def Ext_compute_with_acyclic
(C : cochain_complex š ā¤) (B : š)
[((quotient š (complex_shape.up ā¤)).obj C).is_bounded_above]
(hC : ā k, ā i > 0, is_zero (((Ext' i).obj (op $ C.X k)).obj B))
(i : ā¤) :
((Ext i).obj (op $ of' C)).obj ((single _ 0).obj B) ā
(((preadditive_yoneda.obj B).right_op.map_homological_complex _).obj C).unop.homology (-i) :=
But I'm quite terrified of proving that this is natural in C
. Especially because the typeclass condition on C
forbids stating this as an isom of functors.
Johan Commelin (May 19 2022 at 14:50):
see for_mathlib/acyclic
if you want to inspect this interactively.
Adam Topaz (May 19 2022 at 14:54):
Nice!
Adam Topaz (May 19 2022 at 14:54):
The preserving coproduct thing is almost done... the only sorry left for that is
instance homological_complex_embed_preserves_coproducts {Ī± : Type v}
{M N : Type*} (cā : complex_shape M) (cā : complex_shape N) (e : cā.embedding cā) :
preserves_colimits_of_shape (discrete Ī±)
(homological_complex.embed e : homological_complex A _ ā„¤ _) := sorry
Adam Topaz (May 19 2022 at 14:55):
(I.e. all the homotopy junk has been removed from the statementt)
Adam Topaz (May 19 2022 at 14:55):
I'll try to finish it off, but I don't have much more lean time today, so I don't know how far I'll get.
Adam Topaz (May 19 2022 at 14:56):
It's near the bottom of for_mathlib/derived/ext_coproducts
, just in case
Last updated: Dec 20 2023 at 11:08 UTC