Combinatorics
Daniel Naylor

Contents

1Set Systems
1.1Shadows
1.2Two total orders on X(r)
1.3Compressions
1.4Intersecting Families
2Isoperimetric Inequalities
2.1Concentration of measure
2.2Edge-isoperimetric inequalities
2.3Inequalities in the grid
2.4The edge-isoperimetric inequality in the grid
3Intersecting Families
3.1t-intersecting families
3.2Modular Intersections
3.3Borsuk’s Conjecture
Index

1 Set Systems

Definition 1 (Set system). Let X be a set. A set system on X (or a family of subsets of X) is a family AP(X).

Notation. We will use the notation

X(r)={AX:|A|=r}.

We call an element of X(r) an r-set. We will usually be using X=[n]={1,,n}, so |X(r)|=nr.

Example.

[4](2)={12,13,14,23,24,34}.

Definition 2 (Discrete cube). Make P(X) into a graph by joining A and B if |AΔB|=1, i.e. if A=B{i} for some i, or vice versa. We call this ths discrete cube Qn (if X=[n]).

Example. Q3:

PIC

In general:

PIC

Alternatively, can view Qn as an n-dimensional unit cube {0,1}n, by identifying e.g. {1,3} with 10100000 (i.e. identify A with 𝟙A, the characteristic function of A).

Example.

PIC

Definition 3 (Chain). Say AP(X) is a chain if A,BA, either AB or BA.

PIC

Example. For example,

A={23,12357,123567}

is a chain.

Definition 4 (Antichain). Say A is an antichain if A,BA, AB, we have AB.

PIC

How large can a chain be? Can achieve |A|=n+1, for example using

A={,1,12,123,,[n]}.

Cannot beat this: for each 0rn, A contains 1 r-set.

How large can an antichain be? Can achieve |A|=n, for example A={1,2,,n}. More generally, can take A=X(r), for any r – best out of these is X(n2).

Can we beat this?

Theorem 5 (Sperner’s Lemma). Assuming that:

Then |A|nn2.

Idea: Motivated by “a chain meets each layer in 1 point, because a layer is an antichain”, we will try to decompose the cube into chains.

PIC

Proof. We’ll decompose P(X) into n12n chains – then done. To achieve this, it is sufficient to find:

We then put these together to form our chains, each passing through X(n2).

PIC

By taking complements, it is enough to prove (i).

Let G be the (bipartite) subgraph of Qn spanned by X(r)X(r+1): we seek a matching from X(r) to X(r+1). For any SX(r), the number of SΓ(S) edges in G is |S|(nr) (counting from below) and |Γ(S)|(r+1) (counting from above).

PIC

Hence, as r<n2,

|Γ(S)||S|(nr)r+1|S|.

Thus by Hall’s Marriage theorem, there exists a matching.

Equality in Sperner’s Lemma? Proof above tells us nothing.

Aim: If A is an antichain then

r=0n|AX(r)|nr1.

PIC

“The percentages of each layer occupied add up to 1.”

Trivially implies Sperner’s Lemma (think about it).

Definition 6 (Shadow). For AX(r) (1rn), the shadow of A is A=AX(r1) defined by, A={BX(r1):AA,BA}.

Example. If A={123,124,134,137}X(3), then A={12,13,23,14,24,34,17,37}X(2).

Proposition 7 (Local LYM). Assuming that:

  • AX(r)

  • 1rn

Then
|A|nr1|A|nr.

“The fraction of the level occupied by A is the fraction for A”.

Remark. LYM = Lubell, Meshalkin, Yamamoto.

Proof. The number of AA edges in Qn is |A|r (counting from above) and is |A|(nr+1) (counting from above). So

|A||A|rnr+1.

But nr1nr=rnr+1, so done.

Equality in Local LYM? Must have that AA, iA, jA have A{i}{j}A. So A= or X(r).

Theorem 8 (LYM Inequality). Assuming that:

Then
r=0n|AX(r)|nr1.

Notation. We will now start writing Ar for AX(r).

Proof 1. “Bubble down with Local LYM”.

Have |An|nn1. Now, An and An1 disjoint (as A is an antichain), so

|An|nn1+|An1|nn1=|AnAn1nn11,

whence

|An|nn+|An1|nn11

by Local LYM.

Now, note (AnAn1) is disjoint from An2 (since A is an antichain), so

|(AnAn1)|nn2+|An2|nn21,

whence

|AnAn1|nn1+|An2|nn2.

(Local LYM) so

|An|nn+|An1|nn1+|An2|nn21.

Continue inductively.

Equality in LYM Inequality? Must have had equality in each use of Local LYM. Hence equality in LYM Inequality needs: max r with Ar has Ar=X(r).

So: equality in Local LYM A=X(r) for some r.

Hence: equality in Sperner’s Lemma if and only if A=X(r)n2 (if n even), and A=X(n2) or A=X(n2).

Proof 2. Choose, uniformly at random, a maximal chain C (i.e. C0C1C2Cn, with |Cr|=r for all r).

PIC

For any r-set A, (AC)=1nr (all r-sets are equally likely). So (C meets Ar)=|Ar|nr (as events are disjoint) and hence

1(C meets A)=r=0n|Ar|nr.

Equivalently: (if you want to lose the intuition about how this works) then: #maximal chains=n!, and #through any fixed r-set=r!(nr)!, hence

r|Ar|r!(nr)!n!.

1.1 Shadows

For AX(r), know |A|rnr+1. Equality is rare – only for A= or X(r). What happens in between?

PIC

In other words, given |A|, how should we choose AX(r) to minimise |A|?

Believable that if |A|=kr then we sholud take A=[k](r).

What if kr<|A|<k+1r?

Believable that should take [k](r) plus some r-sets in [k+1](r). For example, for AX(r) with |A|=83+42, take A=[8](3){9B:B[4](2)}.

1.2 Two total orders on X(r)

Let A and B be distinct r-sets: say A=a1,,ar, B=b1,,br where a1<<ar and b1<<br.

Say that A<B in the lexicographic (or lex) ordering if for some j we have ai=bi for i<j and aj<bj.

Slogan: “Use small elements” (“dictionary order”).

Example. lexicographic on [4](2): 12,13,14,23,24,34.

lexicographic on [6](3): 123,124,125,126,134,135,136,145,146,156,234,235,236,245,256,345, 346,356,456.

Say that A<B in the colexicographic (or colex) ordering if for some j we have ai=bi for all i>j and aj<bj.

Slogan: “Avoid large elements” (note that this is not quite the same as “use small elements”, which is what we had before).

Example. colexicographic on [4](2): 12,13,23,14,24,34.

colexicographic on [6](3): 123,124,134,234,125,135,235,145,245,345,126,136,236,146,246,346, 156,256,356,456.

Note that, in colexicographic, [n1](r) is an initial segment (first t elements, for some t) of [n](r).

This is false for lex.

So we could view colexicographic as an enumeration of (r).

Remark. A<B in colexicographic if and only if Ac<Bc in “lexicographic with ground set order reversed”.

Aim: colexicographic initial segments are best for , i.e. if AX(r) and CX(r) is the initial segment of colexicographic with |C|=|A|, then |C||A|.

In particular, |A|=kr|A|kr1.

1.3 Compressions

Idea: try to transform AX(r) into some AX(r) such that:

Ideally, we’d like a family of such ‘compressions’: AAAAB such that either B=C or B is so similar to C that we can directly check that |B||C|.

colexicographic prefers 1 to 2” inspires:

Definition 9 (ij-compression). Fix 1i<jn. The ij-compression Cij is defined as follows:

For AX(r), set

Cij(A)={Aijif jAiAAotherwise,

and for AX(r), set

Cij(A)={Cij(A):AA}{AA:Cij(A)A}.

Note that the second part of the union in Cij(A) is because we need to make sure that we “replace j by i where possible”.

PIC

Example. If A={123,134,234,235,146,567} then C12(A)={123,134,234,135,146,567}.

So Cij(A)X(r), and |Cij(A)|=|A|.

Say A is ij-compressed if Cij(A)=A.

Lemma 10. Assuming that:

  • AX(r)

  • 1i<jn

Then |Cij(A)||A|.

Proof. Write A for Cij(A). Let BAA. We’ll show that iB, jB and BjiAA. [Then done].

PIC

Have BxA for some x, with BxA (as BA). So iBx, jBx, and (Bx)jiA.

Cannot have x=i, else (Bx)ji=Bj, giving BA, contradiction.

Hence we have iB, jB.

Also, BjiA, since (Bx)jiA.

Suppose BjiA: so (Bji)yA for some y. Cannot have y=i, else BjA – so BjA (as jBj), contradicting BA. Hence j(Bji)y and i(Bji)y.

Whence both (Bji)y and By belong to A (by definition of A), contradicting BA.

Remark. Actually showed that Cij(A)CijA.

Definition 11 (Left-compressed). Say AX(r) is left-compressed if Cij(A)=A for all i<j.

Corollary 12. Let AX(r). Then there exists a left-compressed BX(r) with |B|=|A| and |B||A|.

Proof. Define a sequence A0,A1, as follows. Set A0=A. Having defined A0,,Ak, if Ak left-compressed then stop the sequence with Ak.

If not, choose i<j such that Ak is not ij-compression, and set Ak+1=Cij(Ak).

This must terminate, because for example AAkiA is strictly decreasing in k.

Final term B=Ak satisfies |B|=|A|, and |B||A| (by Lemma 10)

Remark.

These compressions only encode the idea “colexicographic prefers i to j (i<j)”, but this is also true for lexicographic.

So we try to come up with more compressions that encode more of what colexicographic likes.

colexicographic prefers 23 to 14” inspires:

Definition 13 (UV-compression). Let U,VX with |U|=|V|, UV= and maxV>maxU. We define the UV-compression as follows: for AX,

CUV(A)={AUVif VAUA=Aotherwise,

and for AX(r), set

CUV(A)={CUV(A):AA}{AA:CUVA}.

Example. If

A={123,124,147,237,238,149},

then

C23,14(A)={123,124,147,237,238,239}.

So CUV(A)X(r), and |CUV(A)|=|A|.

Say A is UV-compressed if CUV(A)=A.

Sadly, we can have |CUV(A)|>|A|:

Example. A={147,157} has |A|=5, but C23,14(A)={237,147} has |C23,14(A)|=6.

Despite this, we at least we do have the following:

Lemma 14. Assuming that:

  • AX(r) is UV-compression for all U,V with |U|=|V|, UV=, maxV>maxU

Then A is an initial segment of colexicographic.

Proof. Suppose not. So there exists A,BX(r) with B<A, in colexicographic but AA, BA.

PIC

Put V=AB, U=BA.

Then |V|=|U|, and U,V disjoint, and maxV>maxU (since max(AΔB)A, by definition of colexicographic).

So CUV(A)=B, contradicting A is UV-compression.

Lemma 15. Assuming that:

  • U,VX

  • |U|=|V|

  • UV=

  • maxU<maxV

  • AX(r)

  • uU vV such that A is (Uu,Vv)-compressed(∗)

Then |CUV(A)||A|.

Proof. Let A=CUV(A). For BAA, we’ll show UB, VB=, and BVUAA. (Then done).

PIC

Have BxA for some x, and BxA, so UBx, V(Bx)=, and (Bx)VUA (by definition of CUV).

If xU: there exists yU such that A is (Ux,Vy)-compressed, so from (Bx)VUA we have ByA – contradicting BA, contradiction.

Thus xU, and so UB, VB=. Certainly BVUA (because (Bx)VUA), so just need to show that BVUA.

Suppose BVUA: so (BVU)wA, for some w. Also have (BVU)wA (for example, as V contained in it).

If wU: know A is (Uw,Vz)-compressed for some zV, so BzA – contradicting B.

If wU: have V(BVU)w, U((BVU)w)=, so by definition of CUV we must have that both (BVU)w and BwA – contradicting BA, a contradiction.

Theorem 16 (Kruskal-Katona). Assuming that:

  • AX(r), 1rn

  • C is the initial segment of colexicographic on X(r) with |C|=|A|

Then |C||A|. In particular: if |A|=kr, then |A|kr1.

Proof. Let Γ={(U,V):|U|=|V|>0,UV=,maxU<maxV}{(,)}. Define a sequence A0,A1, of set systems in X(r) as follows:

Must terminate, as AAkiA2i is strictly decreasing. The final term B=Ak satisfies |B|=|A|, |B||A| and is UV-compressed for all (U,V)Γ.

So B=C by Lemma 14.

Remark.

For AX(r), 0rn, the upper shadow of A is

+A={Ax:AA,xA}X(r+1).

Corollary 17. Let AX(r), where 0rn, and let C be the initial segment of lexicographic on X(r) with |C|=|A|. Then |+A||+C|.

Proof. From Kruskal-Katona, since A<B in colexicographic if and only if Ac<Bc in lexicographic with ground-set order reversed.

Note that the shadow of an initial segment of colexicographic on X(r) is an initial segment of colexicographic on X(r1) – as if C={AX(r):Aa1ar in colexicographic} then C={BX(r1):Ba2ar in colexicographic}.

PIC

This fact gives:

Corollary 18. Let AX(r), and C is the initial segment of colexicographic on X(r) with |C|=|A|. Then |tC||tA| for all 1tr.

Proof. If |tC|tA|, then |t+1C||t+1A|, because tC is an initial segment of colexicographic. Done by induction.

Note. If |A|=kr, then |tA|krt.

Remark. Proof of Kruskal-Katona used Lemma 14 and Lemma 15, but not Lemma 10 or Corollary 12.

1.4 Intersecting Families

Say AP(X) intersecting if AB for all A,BA.

How large can an intersecting family be? Can have |A|=2k1, by taking A={A:1A}.

Proposition 19. Assuming that:

Then |A|2k1.

Proof. For any AX, at most one of A,Ac can belong to A.

Note. Many other extremal examples. For example, for n odd take {A:|A|>k2}.

What if AX(r)?

If r>n2, take A=X(r).

If r=n2: just choose one of A,Ac for all AX(r): gives |A|=12nr.

So interesting case is r<n2.

Could try A={AX(r):1A}. Has size n1r1=rnnr (while this identity can be verified by writing out factorials, a more useful way of observing it is by noting that (random r-set contains 1)=rn).

Could also try B={AX(r):|A{1,2,3}|2}.

Example. n=8, r=3. Then |A|=72=21 and

|B|=1|B[3]|=3+3251|B[3]|=2=16<21.

Theorem 20 (Erdos-Ko-Rado Theorem). Assuming that:

Then |A|n1r1.

Proof 1 (“Bubble down with Kruskal-Katona”). Note that ABABc.

PIC

Let A¯={Ac:AA}X(nr). Have n2rA¯ and A are disjoint families of r-sets.

Suppose |A|>n1r1. Then |A¯|=|A|>n1r1=n1nr. Whence by Kruskal-Katona we have |n2rA¯|n1r.

So |A|+|n2rA¯|>n1r1+n1r=nr, a contradiction.

Remark. Calculation at the end had to give the right answer, as the calculations would all be exact if A={AX(r):1A}.

Proof 2. Pick a cyclic ordering of [n] i.e. a bijection c:[n]n.

PIC

How many sets in A are intervals (r consecutive elements) in this ordering?

Answer: r. Because say C1,,CrA. Then for each 2i1, at most one of the two intervals CiCi+1Ci+r1 and CirCir+1Ci1 can belong to A (subscrpits are modulo n).

For each r-set A, in how many of the n! cyclic orderings is it an interval?

Answer: nr!(nr)! (n= where, r!= order inside A, (nr)!= order outside A).

Hence  A|nr!(nr)!n!r, i.e. |A|n!rnr!(nr)!=n1r1.

Remark.

2 Isoperimetric Inequalities

“How do we minimise the boundary of a set of given size?”

Example. Among all subsets of 2 of given area, the disc minimises the perimeter.

PIC

Among all subsets of 3of given volume, the solid sphere minimises the surface area.

PIC

Among all subsets of S2 of given surface area, the circular arc has the smallest perimeter.

PIC

Definition (Boundary in a graph). For a set A of vertices of a graph G, the boundary of A is

b(A)={xG:xA,xyE for some yA}.

Example. Here, if A={1,2,4}, then b(A)={3,5}.

PIC

Definition (Isoperimetric inequality). An isoperimetric inequality on G is an inequality of the form

|b(A)|f(|A|)AG,

for some function f.

Definition (Neighbourhood). Often simpler to look at the neighbourhood of A: N(A)=Ab(A). So

N(A)={xG:d(x,A)1}.

A good example for A might be a ball B(x,r)={yG:d(x,y)r}. What happens for Qn?

Example. |A|=4 in Q3.

PIC

Good guess that balls are best, i.e. sets of the form B(,r)=X(r)=X(0)X(1)X(r).

What if |X(r)|<|A|<|X(r+1)|?

Guess: take A with X(r)<A<X(r+1). If A=X(r)B, where BX(r+1), then b(A)=(X(r+1)B)+B. So we’d take B to be an initial segment of lexicographic (by Kruskal-Katona).

This suggests...

In the simplicial ordering on P(X), we set x<y if either |x|<|y| or |x|=|y| and x<y in lexicographic.

Aim: initial segments of simplicial ordering minimise the boundary.

Definition (i-sections). For AP(X) and 1in, the i-sections of A are the families A(i),A+(i)P(Xi) given by:

A(i)={xA:ix}A+(i)={xi:xA,ix}

The i-compression of A in the family Ci(A)P(X) given by:

PIC

Example.

PIC

Certainly |Ci(A)|=|A|. Say A is i-compressed if Ci(A)=A. Also, Ci(A) “looks more like” a Hamming ball than A does.

Here, a Hamming ball is a family A with X(r)AX(r+1), for some r.

Theorem 1 (Harper’s Theorem). Assuming that:

Then |N(A)||N(C)|. In particular, if |A|=i=0rni then |N(A)|i=0r+1ni.

PIC

Remark.

Proof. Induction on n: n=1is trivial.

Given n>1, and AQn, and 1in.

Claim: |N(Ci(A))||N(A)|.

Proof of claim: Write B for Ci(A). We have

N(A)=N(A)A+N(A)+=N(A+)A

and of course

N(B)=N(B)B+N(B)+=N(B+)B

Now, |B+|=|A+| and |N(B)||N(A)| (by the induction hypothesis). But B+ is an initial segment of simplicial ordering, and N(B) is an initial segment of simplicial ordering (as neighbourhood of initial segment is an initial segment).

So then B+ and N(B) are nested (one conatined in the other). Hence |N(B)||N(A)|. Similarly, |N(B)+||N(A)+|.

Hence |N(B)||N(A)|, which completes the proof of our claim.

Define a sequence A0,A1,Qn as follows:

Must terminate, because xAk(position of x in simplicial ordering) is strictly decresing.

The final family B=Ak satisfies |B|=|A|, |N(B)||N(A)|, and is i-compressed for all i. Does B i-compressed for all i imply that B is an initial segment of simplicial ordering? (If yes, then B=C and we are done).

Sadly, no. For example in Q3 can take {,1,2,12}:

PIC

However:

Lemma 2. Assuming that:

Then one of the following is true:
  • either n is odd, say n=2k+1, and B=X(k){k+2,k+3,,2k+1}{1,2,,k+1}

  • or n is even, say n=2k, and B=X(<k){xX(k):1x}{1,k+2,k+3,,2k}{2,3,4,,k+1}.

For the even case: “Remove the last k-set with 1, and add the first k-set without 1.”

PIC

After we prove this, we will have solved our problem, as in each case we certainly have |N(B)||N(C)|.

Proof. Since B is not an initial segment of simplicial ordering, there exists x<y (in simplicial ordering) with xB, yB.

PIC

For each 1in: cannot have ix, iy (as B is i-compressed). Also cannot have ix, iy for the same reason.

So x=yc.

Thus: for each yB, there exists at most one earlier x with xB (namely x=yc). Similarly, for each xB there is at most one later y with yB (namely y=xc).

PIC

So B={z:zy}{x}, with x the predessor of y and x=yc.

Hence if n=2k+1 then x is the last k-set, and if n=2k then x is the last k-set with 1.

Proof of Theorem 1. Done by above.

Remark.

For AQn and t=1,2,3,, the t-neighbourhood of A is A(t)=Nt(A)={xQn:d(x,A)t}.

PIC

Corollary 3. Let AQn with |A|i=0rni. Then

|A(t)|i=0r+tni

for all tnr.

Proof. Theorem 1 with induction on t.

To get a feeling for the strength of Corollary 3, we’ll need some estimates on things like i=0rni.

PIC

“Going 𝜀n standard deviations away from the mean n2.”

Proposition 4. Assuming that:

  • 0<𝜀<14

Then
i=0(12𝜀)nni1𝜀e𝜀2n22n.

“For 𝜀 fixed, n, this is an exponentially small fraction of 2n.”

Proof. For i(12𝜀)n:

ni=niini+1,

so

ni1ni=ini+1(12𝜀)n(12+𝜀)n=12𝜀12+𝜀=12𝜀12+𝜀12𝜀.

Hence

i=0(12𝜀)nni12𝜀n(12𝜀)n

(sum of a geometric progression).

Same argument tells us that

n(12𝜀)nn(12𝜀2)n(12𝜀2)𝜀n21-1 from the  stuff2n2(1𝜀)𝜀n22n2e𝜀2n2as 1𝜀e𝜀

Thus

i=0(12𝜀)nni12𝜀2e𝜀2n22n.

Theorem 5. Assuming that:

  • 0<𝜀<14

  • AQn

  • |A|2n12

Then |A(𝜀n)|2n12𝜀e𝜀2n2.

12-sized sets have exponentially large 𝜀n-neighbourhoods.”

Proof. Enough to show that if 𝜀n an integer then

|A(𝜀n)|2n11𝜀e𝜀2n2.

PIC

Have |A|i=0n21ni, so by Harper’s Theorem, we have |A(𝜀n)|i=0n21+𝜀nni, so

|A(𝜀n)c|i=n2+𝜀nnni=i=0n2𝜀nni1𝜀e𝜀2n22n.

Remark. Same would show, for “small” sets:

|A|2n2𝜀e𝜀2n2|A(2𝜀n)|2n12𝜀e𝜀2n2.

2.1 Concentration of measure

Say f:Qn is Lipschitz if |f(x)f(y)|1 for all x,y adjacent.

For f:Qn, say M is a Lévy mean or median of f if

|{xQn:f(x)M}|2n1

and

|{xQn:f(x)M}|2n1

Now ready to show “every well-behaved function on the cube Qn is roughly constant nearly everywhere”.

Theorem 6. Assuming that:

Then
|{x:|f(x)M|𝜀n}|2n14𝜀e𝜀2n2

for any 0<𝜀<14.

Note. This is the “concentration of measure” phenomenon.

PIC

Proof. Let A={x:f(x)M}. Then |A|2n12, so

|A(𝜀n)|2n12𝜀e𝜀2n2.

ut f is Lipschitz, so xA(𝜀n) implies f(x)M+𝜀n. Thus

|{x:f(x)M+𝜀n}|2n12𝜀e𝜀2n2.

Similarly,

|{x:f(x)M𝜀n}|2n12𝜀e𝜀2n2.

Hence

|{x:M𝜀nf(x)M+𝜀n}|2n14𝜀e𝜀2n2.

Let G be a graph of diameter D (D=max{f(x,y):x,yG}).

Definition (α(G,𝜀)). Write

α(G,𝜀)=max{1|A(𝜀D)||G|:AG,|A||G|12}.

So α(G,𝜀) small says “12-sized sets have large 𝜀D-neighbourhoods”.

Definition (Levy family). Say a sequence of graphs is a Lévy family if α(Gn,𝜀)0 as n, for each 𝜀>0.

So Theorem 5 tells us that the sequence (Qn) is a Lévy family – even a normal Lévy family, meaning α(Gn,𝜀) grows exponentially small in n, for each 𝜀>0.

So have concentration of measure for any Lévy family.

Many naturally-occurring families of graphs are Lévy families.

Example. (Sn), where Sn is made into a graph by joining σ to σ if σσ1 is a transposition.

Can define α(X,𝜀) similarly for any metric measure space X (of finite measure and finite diameter).

Example. (Sn) is a Lévy family.

PIC

Two ingredients:

We deduced concentration of measure from an isoperimetric inequality.

Conversely:

Proposition 7. Assuming that:

  • t, α and G are such that for any Lipschitz function f:G with median M we have

    |{xG:|f(x)M|>t}||G|α,

Then for all AG with |A||G|12, we have |A(t)||G|1α.

Proof. The function f(x)=d(x,A) is Lipschitz, and has 0 as a median, so

|{xG:xA(t)}||G|α.

2.2 Edge-isoperimetric inequalities

For a subset A of vertices of a graph G, the edge-boundary of A is

eA=A={xyE:xA,yA}.

PIC

An inequality of the form: |A|f(|A|) for all AG is an edge-isoperimetric inequality on G.

What happens in Qn? Given |A|, which AQn should we take, to minimise |A|?

Example. |A|=4 in Q3:

PIC

This suggests that maybe subcubes are best.

What if AQn? with 2k<|A|<2k+1? Natural to take A=P([k]){some stuff containing k+1}. Suppose we are in Q4, and considering |A|>23, eg |A|=12. We might take the whole of the bottom layer, and then stuff in the upper layer. Note that the size of the boundary will be the number of up edges (which is 1223, a constant), plus the number of edges in the top layer. So we just want to minimise the number of edges in the top layer, i.e. find AQ3 with |A| with minimal boundary.

PIC

So we define: for x,yQn, xy, say x<y in the binary ordering on Qn if maxxΔyy. Equivalently, x<y if and only if ix2i<iy2i. “Go up in subcubes”.

Example. In Q3: ,1,2,12,3,13,23,123.

For AQn, 1in, we define the i-binary compression Bi(A)Qn by giving its i-sections:

(Bi(A))(i)=initial segment of binary on P(Xi) of size |A(i)|(Bi(A))+(i)=initial segment of binary on P(Xi) of size |A+(i)|

so |Bi(A)|=|A|. Say A is i-binary compressed if Bi(A)=A.

PIC

Theorem 8 (Edge-isoperimetric inequality in Qn). Assuming that:

  • AQn

  • let C the initial segment of binary on Qn with |C|=|A|

Then |C||A|. In particular: if |A|=2k then |A|2k(nk).

Remark. Sometimes called the “Theorem of Harper, Lindsey, Bernstein & Hart”.

Proof. Induction on n. n=1 trivial.

For n>1, AQn, 1in:

Claim: |Bi(A)||A|.

Proof of claim: write B for Bi(A). .image Have

|∂A| = |∂(A  )| +|∂(A  )|+ |A  ΔA  |
       ◟-◝−◜-◞  ◟--◝+◜-◞  ◟-+◝◜-−◞
      downstairs  upstairs    across
Also

|B|=|(B)|+|(B+)|+|B+ΔB|.

Now, |(B)||(A)| and |(B+)||(A+)| (induction hypothesis). Also, the sets B+ and B are nested (one is contained inside the other), as each is an initial segment of binary on P(Xi).

Whence we certainly have |B+ΔB||A+ΔA|. So |B||A|.

Define a sequence A0,A1,Qn as follows: set A0=A. Having defined A0,,Ak, if Ak is i-binary compressed for all n then stop the sequence with Ak. If not, choose i with Bi(A)A and put Ak+1=Bi(Ak). Must terminate, as the function kxAk(position of x in binary) is strictly decreasing.

The final family B=Ak satisfies |B|=|A|, |B||A|, and B is i-binary compressed for all i.

Note that B need not be an initial segment of binary, for example {,1,2,3}Q3.

However:

Lemma 9. Assuming that:

Then B=P(n1){1,2,3,,n1}{n} (“downstairs minus the last point, plus the first upstairs point”).

PIC

(Then done, as clearly |B||C|, since C=P(n1)).

Proof. As B not an initial segment, there exists x<y with xB, yB. Then for all i: cannot have ix,y, and cannot have ix,y (as B is i-binary compressed).

Thus for each yB, there exists at most 1 earlier xB (namely x=yc). Also for each xB there is at most one later yB (namely y=xc).

Then x and y adjacent (since y is the unique element in B after x, and x is the unique element not in B before y).

So B={z:zy}{x}, where x is the predecessor of y and y=xc.

So must have y={n}.

This concludes the proof of Theorem 8.

Remark. Vital in the proof of Theorem 8, and of Theorem 1, that the extremal sets (in dimension n1) were nested.

The isoperimetric number of a graph G is

i(G)=min{|A||A|:AG,|A||G|12}.

|A||A| is the “average out-degree of |A|”.

Corollary 10. i(Qn)=1.

Proof. Taking A=P(n1), we show i(Qn)1 (as |A||A|=2n12n=12).

To show i(Qn)12, just need to show that if C is an initial segment of binary with |C|2n1 then |C||C|.

But CP(n1), so certainly |C||C|.

2.3 Inequalities in the grid

For any k=2,3,, the grid is the graph on [k]n in which x is joined to y if for some i we have xj=yj for all ji and |xiyi|=1.

“distance is l1-distance”.

Example. [4]2

PIC

Note that for k=2 this is exactly Qn.

Do we have analogues of Theorem 1 and Theorem 8 for the grid?

Starting with vertex-isoperimetric: which sets A[k]n (of given size) minimise |N(A)|?

Example. In [k]2:

PIC

For A: |b(A)|r2|A|.

For B: |b(B)|=2r=2|B|.

This suggests we “go up in levels” according to |x|=i=1n|xi| – e.g. we’d take {x[k]n:|x|r}.

What if |{x[k]n:|x|r}|<|A|<|{x[k]n:|x|r+1}?

Guess: take A={x[k]n:|x|r} plus some points with |x|=r+1, but which points?

Example. In [k]3:

PIC

so “keep x1 large”.

This suggests in the simplicial order on [k]n, we set x<y if either |x|<|y| or |x|=|y| and xi>yi, where i=min,cbj:xjyj}.

Note. Agrees with the previous definition of simplicial ordering when k=2.

Example. On [3]2: (1,1), (2,1), (1,2), (1,1), (2,2), (1,3), (3,2), (2,3), (3,3).

PIC

On [4]3: (1,1,1), (2,1,1), (1,2,1), (1,1,2), (3,1,1), (2,2,1), (2,1,2), (1,3,1), (1,2,2), (1,1,3), (4,1,1), (3,2,1), …

r A[k]n (n2), and 1in, the i-sections of A are the sets A1,,Ak (or A1(i),,Ak(i)) as a subset of [k]n1 defined by:

At={x[k]n1:(x1,x2,,xi1,t,xi,xi+1,,xn1)A},

for each 1tk.

PIC

The i-compression of A is Ci(A)[k]n is defined by giving its i-sections:

Ci(A)t=initial segment of [k]n1 of size |At|, for each 1tk.

Thus |Ci(A)|=|A|.

Say A is i-compressed if Ci(A)=A.

Theorem 11 (Vertex-isoperimetric inequality in the grid). Assuming that:

Then |N(C)||N(A)|. In particular, if |A||{x:|x|r}| then |N(A)||{x:|x|r+1}|.

Proof. Induction on n. For n=1 it is trivial: if A[k]1,[k]1, then |N(A)||A|+1=|N(C)|.

Given n>1 and A[k]n: fix 1in.

Claim: |N(Ci(A)||N(A)|.

Proof of claim: write B for Ci(A). For any 1tk, we have

N(A)t=N(At)from xi=tAt1from xi=t1At+1from xi=t+1.

PIC

(where A0,Ak+1=).

Also,

N(B)t=N(Bt)Bt1Bt+1.

Now, |Bt1|=|At1| and |Bt+1|=|At+1|, and |N(Bt)||N(At)| (induction hypothesis). But the sets Bt1, Bt+1, N(Bt) are nested (as each is an initial segment of simplicial order on [k]n1).

Hence |N(B)t||N(A)t| for each t. Thus |N(B)||N(A)|.

Among all B[k]n with |B|=|A| and |N(B)||N(A)|, pick one that minimises the quantity xBposition of x in simplicial order.

Then B is i-compressed for all i. Note however, that this time we will make use of this minimality property of B for more than just deducing that B is i-compressed for all i.

Case 1: n=2. What we know is precisely that B is a down-set (A[k]n is a down-set if xA, yixi iyA)

PIC

Let r=min{|x|:xB} and s=max{|x|:xB}. May assume rs, since r=s+1 implies B={x:|x|r1} would imply B=C.

PIC

If r=s: then {x:|x|r1}B{x:|x|r}. So clearly |N(B)||N(C)|.

PIC

If r<s: cannot have {x:|x|=s}B, because then also {x:|x|=r}B (as B is a down-set).

PIC

So there exists y,y with |y|=|y|=s, yB, yB and y=y±(e1e2) (e1=(1,0), e2=(0,1)).

Similarly, cannot have {x:|x|=r}B=, because then {x:|x|=s}B= (as B is a down-set). So there exists x,x with |x|=|x|=r, xB, xB and x=x±(e1en). Now let B=B{x}{y}. From B we lost 1 point in the neighbourhood (namely z in the picture), and gained 1 point (the only point that we can possibly gain is w), so |N(B)||N(B)|. This contradicts minimality of B. This finishes the two dimensional case.

Case 2: n3. For any 1in1 and any xB with xn>1, xi<k. Have xrn+eiB (as B is j-compressed for any j, so apply with some ji,n). So, considering the n-sections of B, we have N(Bt)Bt1 for all t=2,,k.

PIC

Recall that N(B)t=N(Bt)Bt+1Bt1. So in fact N(B)t=Bt1 for all t2. Thus

|N(B)|=|Bk1|level k+|Bk2|level k1++|B1|level 2+|N(B1)|level 1=|B||Bk|+|N(B1)|.

Similarly,

|N(C)|=|C||Ck|+|N(C1)|.

So to show |N(C)||N(B)|, enough to show that |Bk||Ck| and |B1||C1|.

|Bk||Ck|: define a set D[k]n as follows: put Dk=Bk, and for t=k1,k2,,1 set Dt=N(Dt1). Then DB, so |D||B|. Also, D is an initial segment of simplicial order. So in fact DC, whence |Bk|=|Dk||Ck|.

|B1||C1|: define a set E[k]n as follows: put E1=B1 and for t=2,3,,k set Et={x[k]n1:N({x})Et1} (Et is the biggest it could be given N(Et)Et). Then EB, so |E||B|. Also, E is an initial segment of simplicial order. So EC, whence |B1|=|E1||C1|.

Corollary 12. Let A[k]n with |A||{x:|x|n}|. Then |A(t)||{x:|x|r+t}| for all t.

Remark. Can check from Corollary 12 that, for k fixed, the sequence ([k]n)n=1 is a Lévy family.

2.4 The edge-isoperimetric inequality in the grid

Which set A[k]n (of given size) should we take to minimise |A|?

Example. In [k]n:

PIC

Suggests squares are best.

However...

PIC

So we have “phase transitions” at |A|=k24 and 3k24 – extremal sets are not nested. This seems to rule out all our compression methods.

And in [k]3?

[a]3(cube)[a]2×[k](square column)[a]×[k]2(half space)complement of square columncomplement of cube

So in [k]n, up to |A|=kn2, we get n1 of these phase transitions!

Note that if A=[a]×[k]nd. Then |A|=dad1knd=d|A|11dknd1.

Theorem 13. Assuming that:

  • A[k]n

  • |A|kn2

Then
|A|min{d|A|11dknd1:1dn}.

“Some set of the form [a]d×[k]nd is best.”

Called the “edge-isoperimetric inequality in the grid”.

The following discussion is non-examinable (until told otherwise).

Proof (sketch). Induction on n. n=1 is trivial.

Given A[k]n with |A|kn2, where n>1:

Wlog A is a down-set (just down-compress, i.e. stamp on your set in direction i for each i). For any 1in, define Ci(A)[k]n by giving its i-sections:

Ci(A)t=extremal set of size |At| in [k]n1,

which will be a set of the form [a]d×[k]n1d, or a complement. Write B=Ci(A). Do we have |B||A|?

PIC

Now, A is a down-set, so

|A|=|A1|++|Ak|horizontal edges+|A1||Ak|vertical edges

and

|B|=|B1|++|Bk|+?

The ? is because B not a down-set, as extremal sets in dimension n1 are not nested.

Indeed, can have |B|>|A|:

PIC

Idea: try to introduce a “fake” boundary : want AA, with = on extremal sets, such that Ci does decrease (then done).

Try A=t|At|+|A1||Ak|. Then A|A| for all A, equality for extremal sets (as equality for any down-set) and Ci(A)A. But: fails for Cj(A) for all ji.

Could try to fix this by defining A=i(|A1(i)||Ak(i)|). Also fails – for example if A is the “outer shell” of [k]n then A=0.

So far, have

|A|AB=t|Bt|+|B1||Bk|=tf(|Bt|)+|B1||Bk|

where f is the extremal function in [k]n1.

Now, f is the pointwise minimum of some functions of the form cx11d and c(kn1x)11d – each of which is a concave function. Hence f itself is a concave function.

PIC

Consider varying |B2|,,|Bk1|, keeping |B2|++|Bk1| constant and keeping |B1||B2||Bk1||Bk|.

We obtain BC, where for some λ,

Ct={B11tλBkλ+1tk

So:

|A|=ABC=λf(|B1|)+(kλ)f(|Bk|)+|B1||Bk|

but C is still not a down-set.

Now vary, |B1|, keeping λ|B1|+(kλ)|Bk| fixed (λ fixed) and |B1||Bk|.

This is a concave function of |B1| – as concave + concave + linear. Hence “make |B1| as small or large as possible”.

i.e. CD, where one of the following holds:

But (miraculously), this D is a down-set!

PIC

Hence

|A|=ABCD=|D|.

So our “compression in direction i” is: AD.

Now finish as before.

Remark. To make this precise, work instead in [0,1]n (and then take a discrete approximation at the end).

End of non-examinable discussion.

Remark. Very few isoperimetric inequalities are known (even approximately).

For example, “isoperimetric in a layer” – in the graph X(r), with x,y joined if |xy|=r1 (i.e. d(x,y)=2 in Qn).

PIC

This is open. Nicest special case is r=n2, where it is conjectured that balls are best – i.e. sets of the form {x[r](r):|x[r]|t}.

PIC

3 Intersecting Families

3.1 t-intersecting families

AP(X) is called t-intersecting if |xy|t for all x,yA.

How large can a t-intersecting family be?

Example. t=2. Could take {x:1,2x} – has size 142n. Or {x:|x|n2+1} – has size 122n.

PIC

Theorem 1 (Katona’s t-intersecting Theorem). Assuming that:

  • AP(X) is t-intersecting

  • n+t even (to make the proof simpler – same proof works for odd)

Then |A||X(n+t2)|.

Proof. For any x,yA: have |xy|t, so d(x,yc)t. So, writing A¯ for {yc:yA}, have d(A,A¯)t – i.e. A(t1) disjoint from A¯. Suppose that |A|>|X(n+t2)|.

Then, by Harper’s Theorem, we have

|A(t1)||X(n+t2(t1))|=|X(nt2+1)|.

But A(t1) disjoint from A¯, which has size >|X(nt2)| contradicting |A(t1)|+|A¯|2n.

What about t-intersecting AX(r)?

Might guess: best is A0={xX(r):[t]x}.

Could also try Aα={xX(r):|x[t+2α]|t+α}, for α=1,2,,rt.

Example. For 2-intersecting in:

Note that |A0| grows quadratically, |A1| linearly, and |A2| constant – so |A0| largest of these for n large.

PIC

Theorem 2. Assuming that:

Then for n sufficiently large, we have |A||A0|=ntrt.

Remark.

Idea of proof: A0 has rt degrees of freedom”.

Proof. Extending A to a maximal t-intersecting family, we must have some x,yA with |xy|=t (if not, then by maximality have that xA, ix, jx, have xjiA – whence A=X(r), contradiction).

May assume that there exists zA with xyz – otherwise all zA have xyz. Whence |A|ntrt=|A0|.

PIC

So each wA must meet xyz in t+1 points. Thus

|A|23rw on xyz(nrt1+nrt2++n0w off xyz).

Note that the right hand side is a polynomial of degree rt1 – so eventually beaten by |A0|.

3.2 Modular Intersections

For intersecting families, we ban |xy|=0.

What if we banned |xy|0(modsomething)?

Example. Want AX(r) with |xy| odd for all distinct x,yA?

Try r odd: can achieve |A|=n12r12, by picture.

PIC

What if, still for r odd, had |xy| even for all distinct x,yA? Can achieve nr+1, by picture.

PIC

This is only linear in n. Can we improve this?

Similarly if r even: For |xy| even for all x,yA, can achieve |A|=n2r2 – picture

PIC

But for |xy| odd for all x,yA (distinct): can achieve nr+1 (as above). Can we improve this?

Seems to be that banning |xy|=r(mod2) forces the family to be very small (polynomial in n, in fact a linear polynomial).

Remarkably, cannot beat linear.

Proposition 3. Assuming that:

  • r is odd

  • AX(r) such that |xy| for each distinct x,yA

Then |A|n.

Idea: Find |A| linearly independent vectors in a vector space of dimension n, namely Qn.

Proof. View P(X) as 2n, the n-dimensional space over 2 (the field of order 2). By identifying x with x¯, its characteristic sequence (e.g. 1011000 for {1,3,4}).

We have (x¯,x¯)0 for each x, as r is odd ((,) is the usual dot-product).

Also, (x¯,y¯)=0 for distinct x,yA (as |xy| even).

Hence the x¯, xA are linearly independent (if λixi¯=0, dot with xj¯ to get λj=0).

Remark. Hence also if AX(r), r even, with |xy| odd for all distinct x,yA, then |A|n+1 – just add n+1 to each xA and apply Proposition 3 with X=[n+1].

Does this modulo 2 behaviour generalise?

Now show: s allowed values for |xy| modulo p implies |A| polynomial of degree s.

Theorem 4 (Frankl-Wilson Theorem). Assuming that:

  • p is prime

  • λ1,,λs (sr)

  • λir(modp) for each i

  • AX(r) such that for all distinct x,yA have |xy|λi(modp) for some i

Then |A|ns.

Remark.

Idea: Try to find |A| linearly independent points in a vector space of dimension ns, by somehow “applying the polynomial (tλ1)(tλs) to |xy|”.

Proof. For each ij, let M(i,j) be the ni×nj matrix, with rows indexed by X(i), columns indexed by X(j), with

M(i,j)xy={1if xy0otherwise

for each xX(i), yX(j).

PIC

Let V be the vector space (over ) spanned by the rows of M(s,r). So dimVns.

For is, consider M(i,s)M(s,r) (note each row belongs to V, as we premultiplied M(s,r) by a matrix). For xX(i), yX(r):

(M(i,s)M(s,r))xy=# of s-sets z with xz and zy={0if xyrisiif xy

So

M(i,s)M(s,r)=risiM(i,r)

so all rows of M(i,r) belong to V.

Let M(i)=M(i,r)M(i,r) (note each row is in V).

For x,yX(r), have

M(i)xy=#i-sets z with zxzy=|xy|i

Write the integer polynomial (tλ1)(tλs) as i=0saiti, with ai – possible because t(t1)(ti+1)=i!ti.

Let M=i=0saiM(i) (each row is in V).

Then for all x,yX(r):

Mxy=iai|xy|i=(|xy|λi)(|xy|λs).

So the submatrix of M spanned by the rows and columns corresponding to the elements of A is

(000000000).

Hence the rows of M corresponding to A are linearly independent over p, so also over , so also over , so also over .

So |A|dimVns.

Remark. Do need p prime. Grolmusz constructed, for each n, a value of r0(mod6) and a family A[n](r) such that for all distinct x,yA we have |xy|0(mod6) with |A|>nclogn log log n. This is not a polynomial in n.

Corollary 5. Let A[n](r) with |xy|r(modp), for each distinct x,yA, where p<r is prime.

Proof. We are allowed p1 values of |xy|(modp), so done by Frankl-Wilson Theorem.

Two n2-sets in [n] typically meet in about n4 points – but |xy| exactly equaling n4 is very unlikely. But remarkably:

Corollary 6. Let p be prime, and let A[4p](2p) have |xy|p for all distinct x,yA (“this is not much of a constraint”). Then |A|24pp1.

Note. 4pp1 is a tiny (exponentially small) proportion of 4p2p. Indeed, nn2c2nn (for some c) whereas nn42en322n.

Proof. Halving |A| if necessary, may assume that no x,xcA (any x[4p](2p)).

Then x,yA distinct implies |xy|0,p, so |xy|0(modp).

So |A|4pp1 by Corollary 5.

3.3 Borsuk’s Conjecture

Let S be a bounded subset of n.

PIC

How few pieces can we break S into such that each piece has smaller diameter than that of S?

The example of a regular simplex in n (n+1 points, all at distance 1) shows that we may need n+1 pieces.

PIC

Conjecture (Borsuk’s conjecture (1920s)). n+1 pieces always sufficient.

Known for n=1,2,3. Also known for S a smooth convex body in n or a symmetric convex body in n (convex means xS implies xS).

However, Borsuk is massively false:

Theorem 7 (Kahn, Kalai 1995). Assuming that:

  • n

Then there exists bounded Sn such that to break S into pieces of smaller diameter we need Cn, for some constant c>1 (not depending on n).

Note.

Proof. We’ll find SQnn – in fact S[n](r) for some r. We have already had two genuine ideas from this sentence: first that we think about having SQn, and second that we go for S[n](r).

Have S[n](r), so x,yS:

xy2=#coordinates where x and y differ=2(r|xy|).

PIC

So seek S with diameter min|xy|=k, but every subset of S with min|xy|>k is very small (hence we will need many pieces).

Identify [n] with the edge-set of K4p, the complete graph on 4p points.

PIC

For each x[4p](2p) let Gx be the complete bipartite graph, with vertex classes x,xc. Let S={Gx:x[4p](2p)}. So S[n](4p2), and |S|=124p2p.

Now

|GxGy|=|xy||xcyc|+|xcy||xyc|=|xy|2+|xcy|2=d2+(2pd)2

where d=|xy|.

PIC

This is minimised when d=p, i.e. when |xy|=p.

Now let SS have smaller diameter than that of S: say S={Gx:xA}. So must have x,yA distinct: |xy|p (else diameter of S is the diameter of S).

Thus

|A|24pp1.

Conclusion: the number of pieces needed is 124p2p24pp1c24ppep824p (for some c). This is (c)p, for some c>1, which is at least (c)n for some c>1.

˙

Index

antichain

boundary

chain

colexicographic

discrete cube

edge-boundary

grid

i-compressed

Hamming ball

i-binary compressed

i-compressed

ij-compression

intersecting

F

left-compressed

lexicographic

Lévy family

Lipschitz

median

neighbourhood

n-section

r-set

shadow

simplicial ordering

simplicial order

set system

t-intersecting

UV-compression

UV-compressed