Documentation

Mathlib.Combinatorics.Additive.Etransform

e-transforms #

e-transforms are a family of transformations of pairs of finite sets that aim to reduce the size of the sumset while keeping some invariant the same. This file defines a few of them, to be used as internals of other proofs.

Main declarations #

TODO #

Prove the invariance property of the Dyson e-transform.

Dyson e-transform #

def Finset.addDysonEtransform {α : Type u_1} [DecidableEq α] [AddCommGroup α] (e : α) (x : Finset α × Finset α) :

The Dyson e-transform. Turns (s, t) into (s ∪ e +ᵥ t, t ∩ -e +ᵥ s). This reduces the sum of the two sets.

Instances For
    @[simp]
    theorem Finset.addDysonEtransform_fst {α : Type u_1} [DecidableEq α] [AddCommGroup α] (e : α) (x : Finset α × Finset α) :
    (Finset.addDysonEtransform e x).fst = x.fst (e +ᵥ x.snd)
    @[simp]
    theorem Finset.mulDysonEtransform_snd {α : Type u_1} [DecidableEq α] [CommGroup α] (e : α) (x : Finset α × Finset α) :
    (Finset.mulDysonEtransform e x).snd = x.snd e⁻¹ x.fst
    @[simp]
    theorem Finset.addDysonEtransform_snd {α : Type u_1} [DecidableEq α] [AddCommGroup α] (e : α) (x : Finset α × Finset α) :
    (Finset.addDysonEtransform e x).snd = x.snd (-e +ᵥ x.fst)
    @[simp]
    theorem Finset.mulDysonEtransform_fst {α : Type u_1} [DecidableEq α] [CommGroup α] (e : α) (x : Finset α × Finset α) :
    (Finset.mulDysonEtransform e x).fst = x.fst e x.snd
    def Finset.mulDysonEtransform {α : Type u_1} [DecidableEq α] [CommGroup α] (e : α) (x : Finset α × Finset α) :

    The Dyson e-transform. Turns (s, t) into (s ∪ e • t, t ∩ e⁻¹ • s). This reduces the product of the two sets.

    Instances For
      theorem Finset.addDysonEtransform.subset {α : Type u_1} [DecidableEq α] [AddCommGroup α] (e : α) (x : Finset α × Finset α) :
      theorem Finset.mulDysonEtransform.subset {α : Type u_1} [DecidableEq α] [CommGroup α] (e : α) (x : Finset α × Finset α) :

      Two unnamed e-transforms #

      The following two transforms both reduce the product/sum of the two sets. Further, one of them must decrease the sum of the size of the sets (and then the other increases it).

      This pair of transforms doesn't seem to be named in the literature. It is used by Sanders in his bound on Roth numbers, and by DeVos in his proof of Cauchy-Davenport.

      def Finset.addEtransformLeft {α : Type u_1} [DecidableEq α] [AddGroup α] (e : α) (x : Finset α × Finset α) :

      An e-transform. Turns (s, t) into (s ∩ s +ᵥ e, t ∪ -e +ᵥ t). This reduces the sum of the two sets.

      Instances For
        @[simp]
        theorem Finset.addEtransformLeft_snd {α : Type u_1} [DecidableEq α] [AddGroup α] (e : α) (x : Finset α × Finset α) :
        (Finset.addEtransformLeft e x).snd = x.snd (-e +ᵥ x.snd)
        @[simp]
        theorem Finset.mulEtransformLeft_fst {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :
        @[simp]
        theorem Finset.mulEtransformLeft_snd {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :
        (Finset.mulEtransformLeft e x).snd = x.snd e⁻¹ x.snd
        @[simp]
        theorem Finset.addEtransformLeft_fst {α : Type u_1} [DecidableEq α] [AddGroup α] (e : α) (x : Finset α × Finset α) :
        def Finset.mulEtransformLeft {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :

        An e-transform. Turns (s, t) into (s ∩ s • e, t ∪ e⁻¹ • t). This reduces the product of the two sets.

        Instances For
          def Finset.addEtransformRight {α : Type u_1} [DecidableEq α] [AddGroup α] (e : α) (x : Finset α × Finset α) :

          An e-transform. Turns (s, t) into (s ∪ s +ᵥ e, t ∩ -e +ᵥ t). This reduces the sum of the two sets.

          Instances For
            @[simp]
            theorem Finset.mulEtransformRight_fst {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :
            @[simp]
            theorem Finset.addEtransformRight_fst {α : Type u_1} [DecidableEq α] [AddGroup α] (e : α) (x : Finset α × Finset α) :
            @[simp]
            theorem Finset.addEtransformRight_snd {α : Type u_1} [DecidableEq α] [AddGroup α] (e : α) (x : Finset α × Finset α) :
            (Finset.addEtransformRight e x).snd = x.snd (-e +ᵥ x.snd)
            @[simp]
            theorem Finset.mulEtransformRight_snd {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :
            (Finset.mulEtransformRight e x).snd = x.snd e⁻¹ x.snd
            def Finset.mulEtransformRight {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :

            An e-transform. Turns (s, t) into (s ∪ s • e, t ∩ e⁻¹ • t). This reduces the product of the two sets.

            Instances For
              @[simp]
              @[simp]
              theorem Finset.addEtransformLeft.fst_add_snd_subset {α : Type u_1} [DecidableEq α] [AddGroup α] (e : α) (x : Finset α × Finset α) :
              (Finset.addEtransformLeft e x).fst + (Finset.addEtransformLeft e x).snd x.fst + x.snd
              theorem Finset.mulEtransformLeft.fst_mul_snd_subset {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :
              (Finset.mulEtransformLeft e x).fst * (Finset.mulEtransformLeft e x).snd x.fst * x.snd
              theorem Finset.mulEtransformRight.fst_mul_snd_subset {α : Type u_1} [DecidableEq α] [Group α] (e : α) (x : Finset α × Finset α) :

              This statement is meant to be combined with le_or_lt_of_add_le_add and similar lemmas.

              This statement is meant to be combined with le_or_lt_of_add_le_add and similar lemmas.