Zulip Chat Archive
Stream: condensed mathematics
Topic: colimits commute with colimits
Johan Commelin (Mar 17 2022 at 13:31):
Do we actually know that colimits commute with colimits? I need to show that A → A^{⊕n}
commutes with filtered colimits, and would like this to be automatic.
Adam Topaz (Mar 17 2022 at 14:43):
The limit version is in category_theory/limit/fubini
. Looks like we don't have the colimit version.
Adam Topaz (Mar 17 2022 at 14:44):
But since you're using biproducts, it might be easier to do a one-off construction.
Adam Topaz (Mar 17 2022 at 14:45):
I can write something up real quick.
Johan Commelin (Mar 17 2022 at 15:00):
@Adam Topaz I've done that part...
Johan Commelin (Mar 17 2022 at 15:00):
But github didn't let me push it
Adam Topaz (Mar 17 2022 at 15:00):
Oh ok.
Johan Commelin (Mar 17 2022 at 15:00):
Now it worked!
Adam Topaz (Mar 17 2022 at 15:00):
Is GH down?
Johan Commelin (Mar 17 2022 at 15:00):
Half an hour ago I got errors
Johan Commelin (Mar 17 2022 at 15:00):
So I first went for a run
Johan Commelin (Mar 17 2022 at 15:02):
bors still seems to be down...
Johan Commelin (Mar 17 2022 at 15:23):
instance eval_functor_preserves_filtered_colimits (BD : data) [preserves_filtered_colimits F] :
preserves_filtered_colimits ((eval_functor F).obj BD) :=
{ preserves_filtered_colimits := by introsI; apply_instance }
This shows that the Q'
-construction preserves filtered colimits.
- It is currently parameterised by a functor
F
. This should be specialized toℤ[_]
later on. We still need to show thatℤ[_]
preserves filtered colimits. - For https://leanprover-community.github.io/liquid/sect0009.html#homology-Qprime we will also need to show that homology commutes with filtered colimits. That's the missing piece to tick off that box.
Johan Commelin (Mar 17 2022 at 15:24):
@Andrew Yang That second • should be well within the reach of your mathematical toolkit.
Johan Commelin (Mar 17 2022 at 15:25):
[And once again, I can't push to github :sad:]
Johan Commelin (Mar 17 2022 at 15:57):
Mirabile dictu, I managed to push a minute ago!
Andrew Yang (Mar 17 2022 at 16:13):
Great! will start looking at them tomorrow
Adam Topaz (Mar 17 2022 at 17:08):
is by definition a left adjoint, so it preserves all colimits for free! (unless you're talking about a different functor?)
Adam Topaz (Mar 17 2022 at 17:11):
I guess what we're actually missing is the fact that the functor from PFPNG
to Condensed Set
can be computed as the colimit of the condensed sets associated to the profinite levels of the given PFPNG.
Johan Commelin (Mar 17 2022 at 17:23):
@Adam Topaz We mostly need to decide which implementation we use. Maybe we need multiple isomorphic versions of ℤ[_]
.
Adam Topaz (Mar 17 2022 at 17:24):
Do we have the CHPNG version of yet?
Johan Commelin (Mar 17 2022 at 17:24):
I think @Damiano Testa made a start on it.
Johan Commelin (Mar 17 2022 at 17:24):
Or actually, he's defining ℤ[T⁻¹][S]
, I think. (For finite S
.)
Damiano Testa (Mar 17 2022 at 17:39):
What I have is mostly contained in Lbar.finsupp_instance
and src/Lbar/kernel_truncate.lean
.
The first file shows that S
-indexed polynomials (in x^1, but viewed as polynomials in x) are a pseudo_normed_group
.
The second file is a beginning of showing that the kernel of the truncation map from Laurent measures to Lbar actually gives rise to S
-indexed polynomials.
Damiano Testa (Mar 17 2022 at 17:40):
And S
is a Fintype
.
Damiano Testa (Mar 17 2022 at 17:41):
(The S
-indexed polynomials are really the tails of the Laurent series.)
Adam Topaz (Mar 17 2022 at 23:09):
I started on the definition of in terms of profinitely filtered pseudo normed groups in the folder free_pfpng
.
The file free_pfpng/basic
has a few very simple sorry's that I don't have time to finish off right now.
Adam Topaz (Mar 18 2022 at 17:03):
I've added the following stub for Prop 2.1 of analytic.pdf
in free_pfpng/main
:
/-- Prop 2.1 of Analytic.pdf -/
def free_pfpng_profinite_iso :
free_pfpng_profinite ⋙
ProFiltPseuNormGrp₁.enlarging_functor ⋙
ProFiltPseuNormGrp.to_CompHausFilt ⋙
CompHausFiltPseuNormGrp.to_Condensed ≅
Profinite_to_Condensed ⋙ CondensedSet_to_Condensed_Ab := sorry
Johan Commelin (Mar 18 2022 at 17:26):
Thanks for attacking this
Johan Commelin (Mar 18 2022 at 17:27):
Should we have
def ProFiltPseuNormGrp₁.to_Condensed :=
ProFiltPseuNormGrp₁.enlarging_functor ⋙
ProFiltPseuNormGrp.to_CompHausFilt ⋙
CompHausFiltPseuNormGrp.to_Condensed
Adam Topaz (Mar 18 2022 at 17:28):
Sure. Maybe as an abbreviation?
Johan Commelin (Mar 21 2022 at 18:10):
Adam Topaz said:
is by definition a left adjoint, so it preserves all colimits for free! (unless you're talking about a different functor?)
We actually need ℤ[-]
as functor Condensed Ab ⥤ Condensed Ab
. So you have to compose with forget
. So I guess you really need to consider filtered colimits, right?
Last updated: Dec 20 2023 at 11:08 UTC