Sets with very small doubling #
For a finset A in a group, its doubling is #(A * A) / #A. This file characterises sets with
- no doubling as the sets which are either empty or translates of a subgroup.
For the converse, use the existing facts from the pointwise API:
∅ ^ 2 = ∅(Finset.empty_pow),(a • H) ^ 2 = a ^ 2 • H ^ 2 = a ^ 2 • H(smul_pow,coe_set_pow). - doubling strictly less than
3 / 2as the sets that are contained in a coset of a subgroup of size strictly less than3 / 2 * #A. - doubling strictly less than
φas the setAsuch thatA * A⁻¹is covered by at most some constant (depending only on the doubling) number of cosets of a finite subgroup ofG.
TODO #
- Do we need versions stated using the doubling constant (
Finset.mulConst)? - Add characterisation of sets with doubling ≤ 2 - ε. See https://terrytao.wordpress.com/2011/03/12/hamidounes-freiman-kneser-theorem-for-nonabelian-groups.
References #
Doubling exactly 1 #
A non-empty set with no doubling is the left translate of its stabilizer.
A non-empty set with no doubling is the left-translate of its stabilizer.
A non-empty set with no doubling is the right translate of its stabilizer.
A non-empty set with no doubling is the right translate of its stabilizer.
Doubling strictly less than 3 / 2 #
If A has doubling strictly less than 3 / 2, then A⁻¹ * A is a subgroup.
Note that this is sharp: A = {0, 1} in ℤ has doubling 3 / 2 and A⁻¹ * A isn't a subgroup.
Instances For
Equations
If A has doubling strictly less than 3 / 2, then there exists a subgroup H of the
normaliser of A of size strictly less than 3 / 2 * #A such that A is a subset of a coset of
H (in fact a subset of a • H for every a ∈ A).
Note that this is sharp: A = {0, 1} in ℤ has doubling 3 / 2 and can't be covered by a subgroup
of size at most 2.
This is Theorem 2.2.1 in [Toi20].
Doubling strictly less than φ #
If A has doubling K strictly less than φ, then A * A⁻¹ is covered by
at most a constant number of cosets of a finite subgroup of G.
Doubling less than 2-ε #
If S is nonempty such that there is A with |S| ≤ |A| such that |A * S| ≤ (2 - ε) * |S|
for some 0 < ε ≤ 1, then there is a finite subgroup H of G of size |H| ≤ (2 / ε - 1) * |S|
such that S is covered by at most 2 / ε - 1 right cosets of H.
Corollary of card_mul_finset_lt_two in the case A = S, giving characterisation of sets of
doubling less than 2 - ε.