Documentation

MulticolorRamsey.KeyLemma

@[reducible, inline]
abbrev N {C : Type} {V : Type u_1} {G : SimpleGraph V} [DecidableRel G.Adj] [DecidableEq C] [Fintype V] (χ : SimpleGraph.EdgeColoring C) (i : C) (x : V) :
Equations
Instances For
    def mymin {V W : Type} [LinearOrder W] (f : VW) (X : Finset V) [nen : Nonempty { x : V // x X }] :
    W
    Equations
    Instances For
      theorem min_const {V : Type} {c : } {f : V} {X : Finset V} (cn : xX, f x = c) [nen : Nonempty { x : V // x X }] :
      c = mymin f X
      theorem min_le_ℕ {V : Type} {f : V} {g : V} {X : Finset V} [nen : Nonempty { x : V // x X }] (le : xX, f x (g x)) :
      mymin f X (mymin g X)
      theorem min_le_mem_ℕ {V : Type} {f : V} {X : Finset V} {v : { x : V // x X }} [Nonempty { x : V // x X }] :
      mymin f X f v
      def pY {r : } {V : Type} [Fintype V] [DecidableEq V] (X Y : Finset V) [nen : Nonempty { x : V // x X }] (χ : SimpleGraph.EdgeColoring (Fin r)) (i : Fin r) :
      Equations
      Instances For
        noncomputable def p {r : } {V : Type} [Fintype V] [DecidableEq V] (X Y : Finset V) [Nonempty { x : V // x X }] (EC : SimpleGraph.EdgeColoring (Fin r)) (i : Fin r) :
        Equations
        Instances For
          def lift {V : Type u_1} {X : Finset V} (X' : Finset { x : V // x X }) :
          Equations
          Instances For
            instance lift.Nonempty {V : Type u_1} {X : Finset V} (X' : Finset { x : V // x X }) [nen : _root_.Nonempty { x : { x : V // x X } // x X' }] :
            theorem tr {V : Type u_1} {X : Finset V} {X' : Finset { x : V // x X }} {p : VProp} (e : aX', p a) (x : V) :
            x lift X'p x
            theorem key {r n : } [Nonempty (Fin r)] (V : Type) [DecidableEq V] [Nonempty V] [Fintype V] {cardV : Fintype.card V = n} (χ : SimpleGraph.EdgeColoring (Fin r)) (X : Finset V) [nenX : Nonempty { x : V // x X }] (Y : Fin rFinset V) (Ypos : ∀ (i : Fin r), 0 < (Y i).card) (α : Fin r) (αpos : ∀ (i : Fin r), 0 < α i) (ppos : ∀ (i : Fin r), 0 < pY X (Y i) χ i) :
            let β := 3 ^ (-4 * r); let C := 4 * r * r; ∃ (l : Fin r) (Λ : ), -1 Λ xX, ∃ (X' : Finset { x : V // x X }) (nx : Nonempty { x : { x : V // x X } // x X' }) (Y' : Fin rFinset V), (∀ (i : Fin r), Y' i N χ i x Y i) β * Real.exp (-C * (Λ + 1)) * X.card X'.card (∀ (i : Fin r), i l(Y' i).card = p X (Y i) χ i * (Y i).card) p X (Y l) χ l + Λ * α l p (lift X') (Y' l) χ l ∀ (i : Fin r), i lp X (Y i) χ i - α i p (lift X') (Y' i) χ i