Zulip Chat Archive
Stream: Carleson
Topic: lemma 7.7.1 forest row-decomposition
Edward van de Meent (Feb 12 2025 at 16:44):
for 7.1.1 7.7.1 i have one sorry left i can't figure out... i can't figure out why the new is -disjoint from the previous ones (in the proof of ∀ x:X, stackSize (t \ ⋃ i < j, t.rowDecomp i : Set _) x ≤ 2 ^ n - j
)
Edward van de Meent (Feb 12 2025 at 16:49):
see here(old) here for my code
Edward van de Meent (Feb 12 2025 at 16:50):
(also beware the code is not cleaned up yet)
Floris van Doorn (Feb 12 2025 at 19:00):
It's very hard to understand where you are in the proof when linking to a Lean formalization, and much easier if you refer to a particular step in the blueprint.
What I think is going on: you want to show that every element x
still occurring in the forest after removing j
rows actually occurs in at least one element of thej
-th row. And you're proving that if this is not the case, you can add a maximal element containing x
to the row contradicting the maximalness of the row. The reason that this new element is disjoint follows from the axioms of the grid, since elements of the grid are comparable or disjoint: carleson#le_or_ge_or_disjoint
Since both u
and t
are maximal elements and not equal, they cannot be comparable.
Does that finish your proof?
PS: you might want to use the order on Grid X
directly, instead of casting it to Set X
, e.g. by using the following in rowDecomp_zornset
∀ u ∈ x, Maximal (· ∈ ((fun x => 𝓘 x : 𝔓 X → Grid X) '' s)) (𝓘 u)
Edward van de Meent (Feb 12 2025 at 20:12):
i think i don't want that order tho? the reason i need this maximality (i think) is because stackSize
refers to the members of the set corresponding with a grid point
Edward van de Meent (Feb 12 2025 at 20:14):
i think that's why the blueprint specifies "... with inclusion maximal ." (emphasis mine)
Edward van de Meent (Feb 12 2025 at 20:19):
(because i seem to recall that this order is not the same as just the inclusion order?)
Floris van Doorn (Feb 12 2025 at 20:19):
The orders are actually quite similar: carleson#Grid.le_def
In particular, every Grid-maximal element should be Set-maximal.
But I think in this proof the difference doesn't really matter
Edward van de Meent (Feb 12 2025 at 20:26):
i guess i'm not quite clear if the definition refers to -disjointness or -disjointness?
Edward van de Meent (Feb 12 2025 at 20:28):
carleson#le_or_ge_or_disjoint seems to refer to the former
Floris van Doorn (Feb 12 2025 at 20:28):
carleson#Grid.le_def talks about elements in , if that's what you're asking.
But I guess we're getting off track. Did the rest of my message solve the gap in your proof?
Edward van de Meent (Feb 12 2025 at 20:31):
Floris van Doorn said:
The reason that this new element is disjoint follows from the axioms of the grid, since elements of the grid are comparable or disjoint: carleson#le_or_ge_or_disjoint
this explains why the new element's image under is disjoint from the images of the previous ones, but as far as i can tell (for the purposes of carleson#TileStructure.Row.pairwiseDisjoint' ) i need to explain why the new element's image under is disjoint from the previous ones
Edward van de Meent (Feb 12 2025 at 20:35):
i.e. the construction says to choose disjoint tiles (under , implied), then the proof that this construction covers everything in says a certain kind of tile must be in there due to maximality of your choice, but then you need to prove that including the new tile still satisfies your constraints
Notification Bot (Feb 12 2025 at 20:38):
13 messages were moved here from #Carleson > Outstanding Tasks, V5 by Edward van de Meent.
Floris van Doorn (Feb 13 2025 at 15:55):
Yes, you're right. I made a mistake last night, confusing tiles and cubes myself.
Floris van Doorn (Feb 13 2025 at 15:55):
I think there is indeed a gap in the proof there. I'll ask my coauthors if they see how to fix it.
Floris van Doorn (Feb 13 2025 at 16:57):
Oops, this was my fault, sorry!
I wrongly translated the definition of Row
into Lean. I should have written that the 𝓘(u)
are disjoint, not the 𝔗(u)
. Also, in the first sentence of the proof of Lemma 7.7.1, the disjointness means that the 𝓘(u)
s are disjoint.
The proof will be almost the same, but now you can use the dyadic property of the cubes ( carleson#le_or_ge_or_disjoint ) in the place where you got stuck
Floris van Doorn (Feb 13 2025 at 16:58):
I just pushed a commit fixing the definition of Row
.
Edward van de Meent (Feb 13 2025 at 17:02):
awesome, indeed that does fix the proof :thumbs_up:
Edward van de Meent (Feb 13 2025 at 19:38):
actually, for this proof, i'd need to be some sort of injective, i think? i have locally proven that indeed, if is in the j
th row and both and have maximal images under (i.e. maximal for the points remaining), their images under are either disjoint or equal... but i'm not sure that i get to conclude that that contradicts ?
Edward van de Meent (Feb 13 2025 at 19:40):
can i somehow prove that this new is in :thinking:
Floris van Doorn (Feb 13 2025 at 22:14):
is definitely not intended to be injective.
Floris van Doorn (Feb 13 2025 at 22:17):
Can you state more precisely where you are in the proof? Are you still on the sentence "Thus it is contained in a cube in with "? What is ?
Edward van de Meent (Feb 14 2025 at 12:05):
Floris van Doorn said:
Since both
u
andt
are maximal elements and not equal, they cannot be comparable.
this is the bit where i get stuck, since technically we're not comparing u
and t
but 𝓘 u
and 𝓘 t
Edward van de Meent (Feb 14 2025 at 12:09):
i.e. we know u
and t
are not equal, but the maximality and disjointness are about 𝓘 u
and 𝓘 t
. I have managed to prove that either 𝓘 u
and 𝓘 t
are disjoint or equal, but i don't know how to get a contradiction in the equal case.
Floris van Doorn (Feb 17 2025 at 08:42):
You're considering the case where there is some x
in 𝓘 u
that is not in 𝓘 t
for any t
in the j
-th row, right? So therefore, 𝓘 u = 𝓘 t
is impossible.
Floris van Doorn (Feb 17 2025 at 08:46):
Edward van de Meent said:
this is the bit where i get stuck, since technically we're not comparing
u
andt
but𝓘 u
and𝓘 t
I believe the order on 𝔓 X
should not be used at all in Lemma 7.7.1. EDIT: I misread what you said, we're in agreement.
Floris van Doorn (Feb 17 2025 at 08:50):
If you're still stuck, please write in English the argument you're giving after the sentence "[...] then it is contained in a maximal such cube." in the proof of Lemma 7.7.1, and where you're stuck.
Edward van de Meent (Feb 17 2025 at 12:53):
Ah, that fixes it (for real this time). Indeed, we get to assume that there exists no such t
and do proof by contradiction! I missed that bit
Edward van de Meent (Feb 17 2025 at 12:55):
My proof is now sorry free locally, I'll polish the proof and then make a PR
Edward van de Meent (Feb 22 2025 at 12:25):
Last updated: May 02 2025 at 03:31 UTC