Zulip Chat Archive
Stream: condensed mathematics
Topic: homology of Q'
Johan Commelin (Jun 09 2022 at 04:57):
In https://leanprover-community.github.io/liquid/sect0008.html#Qprime-Cond we have the statement
for torsion-free condensed abelian groups . The way you prove this is by writing as a filtered colimit of fg free objects, and then noting that and both commute with filtered colimits and direct sums. commutes with direct sums when viewed as a functor to the homotopy category because of the homotopy condition in BD packages.
I don't see any obstructions to formalizing this. But I have a maths question: what we really need is the fact that this is also natural in . More precisely: if is an endomorphism, and we push it through the functors on the left, why do we end up with on the right?
Johan Commelin (Jun 09 2022 at 04:57):
It's the only reasonable candidate, but I couldn't figure out a precise proof easily.
Peter Scholze (Jun 09 2022 at 05:06):
About the proof: You first prove the result on presheaves -- for extremally disconnected -- and for this you write in the way described in Johan's message. ( itself is very much not a filtered colimit of fg free objects in general.)
Johan Commelin (Jun 09 2022 at 05:08):
Aah, good point. Yes, my verbal summary of the strategy was a bit too fast.
Peter Scholze (Jun 09 2022 at 05:08):
To get functoriality: Maybe it's easier if you first describe the map, at least on elementary tensors? It sends to the image of under the map induced by the map sending to .
Adam Topaz (Jun 10 2022 at 19:58):
@Johan Commelin do we have an established way to talk about torsion-free (condensed) abelian groups?
Johan Commelin (Jun 10 2022 at 20:09):
Nope, I don't think there is anything about torsion free. Although mathlib does have something about torsion, but I'm not sure that's too relevant.
Adam Topaz (Jun 11 2022 at 04:32):
I added some work in progress toward this lemma in for_mathlib/AddcommGroup
near the bottom.
A few sorries there are very easy... any help would be much appreciated!
Adam Topaz (Jun 11 2022 at 13:57):
Adam Topaz said:
Johan Commelin do we have an established way to talk about torsion-free (condensed) abelian groups?
For future reference, I used docs#no_zero_smul_divisors because that's what's used in docs#module.free_of_finite_type_torsion_free
Adam Topaz (Jun 11 2022 at 23:51):
This is now sorry-free in for_mathlib/AddCommGroup
lemma is_iso_of_preserves_of_is_tensor_unit {𝓐 : Type u'} [category.{u} 𝓐] [preadditive 𝓐]
(F G : AddCommGroup ⥤ 𝓐)
[F.additive]
[G.additive]
[limits.preserves_filtered_colimits F]
[limits.preserves_filtered_colimits G]
(η : F ⟶ G)
(U : AddCommGroup)
(hU : U.is_tensor_unit)
[hη : is_iso (η.app U)]
(A : AddCommGroup.{u})
[no_zero_smul_divisors ℤ A] :
is_iso (η.app A) := ...
where
def is_tensor_unit (A : AddCommGroup.{u}) : Prop :=
∃ a : A, ∀ (B : AddCommGroup.{u}), function.bijective
(λ f : A ⟶ B, (f : A → B) a)
This way we don't need to make a choice about what tensor unit we choose.
Last updated: Dec 20 2023 at 11:08 UTC