Zulip Chat Archive
Stream: Is there code for X?
Topic: is_iso dist triang
Adam Topaz (Feb 21 2022 at 20:45):
I just want to verify that we don't have the following lemma
https://stacks.math.columbia.edu/tag/014A
before I start using docs#category_theory.abelian.is_iso_of_is_iso_of_is_iso_of_is_iso_of_is_iso :)
Adam Topaz (Feb 21 2022 at 20:59):
Ping @Andrew Yang @Johan Commelin @Matthew Ballard
Matthew Ballard (Feb 21 2022 at 20:59):
I just thought that name was a joke...
Adam Topaz (Feb 21 2022 at 20:59):
That's the five lemma :rofl:
Andrew Yang (Feb 21 2022 at 21:00):
I don’t think we have that yet
Adam Topaz (Feb 21 2022 at 21:02):
Okay. I'll prove it later today. I already added the stub to LTE.
Matthew Ballard (Feb 21 2022 at 21:02):
I think you need to know that is homological as a prereq to stacks#014A
Adam Topaz (Feb 21 2022 at 21:03):
We did that last week!
Matthew Ballard (Feb 21 2022 at 21:03):
Is it in mathlib? :stuck_out_tongue:
Adam Topaz (Feb 21 2022 at 21:03):
Ah, no.
Adam Topaz (Feb 21 2022 at 21:05):
@Andrew Yang how's it going with projective replacements? Did you see some of the stuff in the recent for_mathlib/derived
folder from LTE?
Matthew Ballard (Feb 21 2022 at 21:06):
I think that is the main missing piece. The rest is Yoneda + repeat 5 is_iso
Andrew Yang (Feb 21 2022 at 21:14):
All the data are constructed but I’m struggling to show that it is quasi iso despite having finished all the diagram chasing parts because of some dependent type issues. I have a busy day tomorrow, so I hope I’ll be able to finish it the day after.
Andrew Yang (Feb 21 2022 at 21:16):
I noticed there’s quite a lot going on in that directory, but I have yet to look into it.
Adam Topaz (Feb 21 2022 at 21:25):
We defined is_quasi_iso
there. It would be useful to know how you formulate boundedness so that I can add that condition to one of the theorems
Andrew Yang (Feb 22 2022 at 00:39):
There’s also docs#quasi_iso that seems to have the same definition.
For boundedness I simply used
“forall i > a, is_iso (0 : X.X i -> 0)”
(sorry, on a phone now)
Adam Topaz (Feb 22 2022 at 00:42):
Ah ok. Yeah, the one in for_mathlib/derived
is for the homotopy category, but it's essentially the same yes.
Last updated: Dec 20 2023 at 11:08 UTC