Zulip Chat Archive
Stream: condensed mathematics
Topic: BD lemma: last line
Johan Commelin (Jun 01 2022 at 09:15):
The last line of the proof of https://leanprover-community.github.io/liquid/sect0008.html#Qprime-prop is
In general, one can pick a two-term free resolution of and use the long exact sequence.
I am now wondering what the smoothest way is to do this in Lean.
The context is the following: Let be an abelian group and a free resolution. Let be a condensed abelian group (which we can assume to be torsion-free). We want to show that vanishes, and we know already that vanishes for free .
I think the easiest way to continue is to show that is short exact, using the fact that is torsion-free. What I really want to avoid is any theoretical properties of Tor
, because we don't have anything about it. What is the cheapest (in terms of ingredients) way to prove (on paper) that a torsion-free abelian group is flat?
Note that we don't even need to show that M ⊗ _
is exact: a direct proof that it sends injective maps between free abelian groups to injective maps is all we need.
Kevin Buzzard (Jun 01 2022 at 09:55):
Torsion-free is a filtered colimit of f.g. free, does that help?
Johan Commelin (Jun 01 2022 at 10:11):
I guess it does
Filippo A. E. Nuccio (Jun 04 2022 at 11:05):
OK, so moving from Kevin's suggestion, this is a strategy I came up with, trying to check what is already in mathlib
:
1) Following Kevin's idea, I reduce to the case where both M, F1 and F2
are finitely generated free abelian groups. Yet, two things are not clear to me here:
1a) Is Kevin's claim already in mathlib
(on in themathlib
folder)?
1b) Same question for "filtered colimit of injections is injective" (aka left-exactness, but I do not know how and if this is implemented)
2) So now I have to prove that if is an injection of finitely generated free abelian groups and is also f. g. free, then is injective. For this, I would use the
lemma foo (f : M →ₗ[R] N) (v : ι → M) (hv : basis ι R M)
(hι : fintype ι)
: function.injective f ↔ linear_independent R (f ∘ v) :=
saying that a linear map is injective iff it sends a basis to a linearly independent set.
3) So I have three bases and of respectively; I can use docs#module.free.tensor to know that is a basis of and I apply to each member. I need to show that the result is a linearly independent set.
4) For this, I would like to adapt some of the results we have for determinants (like the first part of docs#linear_independent) to show that if a determinant is non-zero, then the set is linearly independent
5) Finally, I would adapt some results from docs#matrix.kronecker to the effect that the matrix representing wrt and is the Kronecker product of the identity and of the matrix representing and hence its determinant is non-zero by the assumption on .
Does it sound a sufficiently down-to-earth plan? I can start working on this soon.
Johan Commelin (Jun 04 2022 at 11:08):
I think you don't even need to do reduction steps for F₁
and F₂
.
If you have a SES 0 → A → B → C → 0
and you tensor it with M
, where M
is a filtered colimit of fg free groups, then you reduce to checking that
- your 1b
- the SES remains injective after tensoring with fg free groups
Johan Commelin (Jun 04 2022 at 11:09):
But tensoring with fg free groups is just taking a suitable direct sum of the objects in the SES, and it should be easy to prove that this remains exact by induction.
Adam Topaz (Jun 04 2022 at 11:10):
I'm not so sure about that last point -- you really need the torsion-freeness assumption for that!
Johan Commelin (Jun 04 2022 at 11:11):
Which point? If you have a SES and you tensor it with ℤ^k
then it remains a SES.
Adam Topaz (Jun 04 2022 at 11:11):
yeah
Johan Commelin (Jun 04 2022 at 11:11):
That's just because ℤ^k
is free, hence flat.
Adam Topaz (Jun 04 2022 at 11:12):
Oh sorry, tensor WITH Z^k, okay yeah that's easy
Johan Commelin (Jun 04 2022 at 11:12):
The torsion-free-ness is used completely in showing that M
is a filtered colimit of fg free groups.
Adam Topaz (Jun 04 2022 at 11:12):
yeah I agree sorry I should have read more carefully
Adam Topaz (Jun 04 2022 at 11:12):
that should indeed just be a simple induction on k
Johan Commelin (Jun 04 2022 at 11:14):
I think I would try to stay in the realm of category theory as long as possible. You should be able to avoid kronecker products completely.
Adam Topaz (Jun 04 2022 at 11:15):
Do we know that tf implies filtered colimit of f.g. free?
Johan Commelin (Jun 04 2022 at 11:16):
Nope, I guess not.
Filippo A. E. Nuccio (Jun 04 2022 at 11:35):
Yes, I guess you are right, we do not need to pick basis for and . I will then first of all try to prove that tf implies filtered colimit of f.g. free, and then prove the lemma by induction on .
Filippo A. E. Nuccio (Jun 06 2022 at 07:37):
Another idea that came to my mind is the following: I fix two free -modules with an injection and a torsion-free . If we can show that is injective, then also is injective, because so is by the torsion-freeness assumption. In order to show that is injective, we can write the arrow as
and therefore the key point becomes to show that (not-necessarily finite dimensional) vector spaces are flat. One proof of this fact goes through proving that they are a cofiltered limit of their finite dimensional subspaces, but then we are basically back at Kevin's suggestion. Is there an easier way to show this flatness of vector spaces directly? According to this thread on MO, it only holds under AC...
Johan Commelin (Jun 06 2022 at 07:42):
I think this requires API about base change of the ring of scalars that we don't have yet.
Filippo A. E. Nuccio (Jun 06 2022 at 07:43):
At which point? We have that the tensor product is associative and commutative and that the tensor prod of two free is free.
Filippo A. E. Nuccio (Jun 06 2022 at 07:44):
If it is about tensoring over instead of over once everything is a v.s., isn't it worth building this API?
Filippo A. E. Nuccio (Jun 06 2022 at 07:45):
I also understand that you want to go straight to the point, but if there was an easier way avoiding the fact that colimits are left exact and that a torsion-free is a filtered colimit of f.g. free, I though it might be at any rate a good trial.
Johan Commelin (Jun 06 2022 at 08:05):
I think it's certainly worth building that API at some point. But I think exhibiting a tf ab group as cofiltered limit of fg free ones shouldn't be too hard, and is also worth building.
Filippo A. E. Nuccio (Jun 06 2022 at 08:06):
OK, I guess you have a clearer picture. I will follow that line. And what about left-exactness of colimits, is it already there (in LTE, perhaps)?
Adam Topaz (Jun 06 2022 at 10:31):
You could use the fact that filtered colimits commute with finite limits (e.g. kernels) which is in mathlib, or just do it by hand since you're working with abelian groups, using the mathlib api for filtered colimits in concrete categories (category_theory/limits/concrete
)
Adam Topaz (Jun 06 2022 at 10:50):
Well, the quickest way is probably to just do things in a totally hands on way with sums of basic tensors. Take an element of the tensor product, write it as a sum of basic tensors to find a f.g. free submodule whose tensor product contains those elements, and use that to reduce to the free case.
Filippo A. E. Nuccio (Jun 08 2022 at 09:08):
Yes, I agree this should be the quickest way. Thanks!
Filippo A. E. Nuccio (Jun 30 2022 at 17:30):
(deleted)
Filippo A. E. Nuccio (Jun 30 2022 at 17:31):
(deleted)
Filippo A. E. Nuccio (Jun 30 2022 at 17:34):
(deleted)
Last updated: Dec 20 2023 at 11:08 UTC