Documentation

Mathlib.Analysis.BoxIntegral.Partition.Split

Split a box along one or more hyperplanes #

Main definitions #

A hyperplane {x : ι → ℝ | x i = a} splits a rectangular box I : BoxIntegral.Box ι into two smaller boxes. If a ∉ Ioo (I.lower i, I.upper i), then one of these boxes is empty, so it is not a box in the sense of BoxIntegral.Box.

We introduce the following definitions.

Main results #

The main result BoxIntegral.Prepartition.exists_iUnion_eq_diff says that any prepartition π of I admits a prepartition π' of I that covers exactly I \ π.iUnion. One of these prepartitions is available as BoxIntegral.Prepartition.compl.

Tags #

rectangular box, partition, hyperplane

def BoxIntegral.Box.splitLower {ι : Type u_1} (I : BoxIntegral.Box ι) (i : ι) (x : ) :

Given a box I and x ∈ (I.lower i, I.upper i), the hyperplane {y : ι → ℝ | y i = x} splits I into two boxes. BoxIntegral.Box.splitLower I i x is the box I ∩ {y | y i ≤ x} (if it is nonempty). As usual, we represent a box that may be empty as WithBot (BoxIntegral.Box ι).

Equations
Instances For
    @[simp]
    theorem BoxIntegral.Box.coe_splitLower {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
    (BoxIntegral.Box.splitLower I i x) = I {y : ι | y i x}
    theorem BoxIntegral.Box.splitLower_le {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
    @[simp]
    theorem BoxIntegral.Box.splitLower_eq_bot {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
    @[simp]
    theorem BoxIntegral.Box.splitLower_eq_self {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
    BoxIntegral.Box.splitLower I i x = I I.upper i x
    theorem BoxIntegral.Box.splitLower_def {ι : Type u_1} {I : BoxIntegral.Box ι} [DecidableEq ι] {i : ι} {x : } (h : x Set.Ioo (I.lower i) (I.upper i)) (h' : optParam (∀ (j : ι), I.lower j < Function.update I.upper i x j) ) :
    BoxIntegral.Box.splitLower I i x = { lower := I.lower, upper := Function.update I.upper i x, lower_lt_upper := h' }
    def BoxIntegral.Box.splitUpper {ι : Type u_1} (I : BoxIntegral.Box ι) (i : ι) (x : ) :

    Given a box I and x ∈ (I.lower i, I.upper i), the hyperplane {y : ι → ℝ | y i = x} splits I into two boxes. BoxIntegral.Box.splitUpper I i x is the box I ∩ {y | x < y i} (if it is nonempty). As usual, we represent a box that may be empty as WithBot (BoxIntegral.Box ι).

    Equations
    Instances For
      @[simp]
      theorem BoxIntegral.Box.coe_splitUpper {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
      (BoxIntegral.Box.splitUpper I i x) = I {y : ι | x < y i}
      theorem BoxIntegral.Box.splitUpper_le {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
      @[simp]
      theorem BoxIntegral.Box.splitUpper_eq_bot {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
      @[simp]
      theorem BoxIntegral.Box.splitUpper_eq_self {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } :
      BoxIntegral.Box.splitUpper I i x = I x I.lower i
      theorem BoxIntegral.Box.splitUpper_def {ι : Type u_1} {I : BoxIntegral.Box ι} [DecidableEq ι] {i : ι} {x : } (h : x Set.Ioo (I.lower i) (I.upper i)) (h' : optParam (∀ (j : ι), Function.update I.lower i x j < I.upper j) ) :
      BoxIntegral.Box.splitUpper I i x = { lower := Function.update I.lower i x, upper := I.upper, lower_lt_upper := h' }

      The partition of I : Box ι into the boxes I ∩ {y | y ≤ x i} and I ∩ {y | x i < y}. One of these boxes can be empty, then this partition is just the single-box partition .

      Equations
      Instances For
        theorem BoxIntegral.Prepartition.mem_split_iff' {ι : Type u_1} {I : BoxIntegral.Box ι} {J : BoxIntegral.Box ι} {i : ι} {x : } :
        J BoxIntegral.Prepartition.split I i x J = I {y : ι | y i x} J = I {y : ι | x < y i}
        theorem BoxIntegral.Prepartition.split_of_not_mem_Ioo {ι : Type u_1} {I : BoxIntegral.Box ι} {i : ι} {x : } (h : xSet.Ioo (I.lower i) (I.upper i)) :

        If x ∉ (I.lower i, I.upper i), then the hyperplane {y | y i = x} does not split I.

        theorem BoxIntegral.Prepartition.coe_eq_of_mem_split_of_mem_le {ι : Type u_1} {I : BoxIntegral.Box ι} {J : BoxIntegral.Box ι} {i : ι} {x : } {y : ι} (h₁ : J BoxIntegral.Prepartition.split I i x) (h₂ : y J) (h₃ : y i x) :
        J = I {y : ι | y i x}
        theorem BoxIntegral.Prepartition.coe_eq_of_mem_split_of_lt_mem {ι : Type u_1} {I : BoxIntegral.Box ι} {J : BoxIntegral.Box ι} {i : ι} {x : } {y : ι} (h₁ : J BoxIntegral.Prepartition.split I i x) (h₂ : y J) (h₃ : x < y i) :
        J = I {y : ι | x < y i}

        Split a box along many hyperplanes {y | y i = x}; each hyperplane is given by the pair (i x).

        Equations
        Instances For
          theorem BoxIntegral.Prepartition.not_disjoint_imp_le_of_subset_of_mem_splitMany {ι : Type u_1} {I : BoxIntegral.Box ι} {J : BoxIntegral.Box ι} {Js : BoxIntegral.Box ι} {s : Finset (ι × )} (H : ∀ (i : ι), {(i, J.lower i), (i, J.upper i)} s) (HJs : Js BoxIntegral.Prepartition.splitMany I s) (Hn : ¬Disjoint J Js) :
          Js J

          Let s : Finset (ι × ℝ) be a set of hyperplanes {x : ι → ℝ | x i = r} in ι → ℝ encoded as pairs (i, r). Suppose that this set contains all faces of a box J. The hyperplanes of s split a box I into subboxes. Let Js be one of them. If J and Js have nonempty intersection, then Js is a subbox of J.

          theorem BoxIntegral.Prepartition.eventually_not_disjoint_imp_le_of_mem_splitMany {ι : Type u_1} [Finite ι] (s : Finset (BoxIntegral.Box ι)) :
          ∀ᶠ (t : Finset (ι × )) in Filter.atTop, ∀ (I J : BoxIntegral.Box ι), J sJ'BoxIntegral.Prepartition.splitMany I t, ¬Disjoint J J'J' J

          Let s be a finite set of boxes in ℝⁿ = ι → ℝ. Then there exists a finite set t₀ of hyperplanes (namely, the set of all hyperfaces of boxes in s) such that for any t ⊇ t₀ and any box I in ℝⁿ the following holds. The hyperplanes from t split I into subboxes. Let J' be one of them, and let J be one of the boxes in s. If these boxes have a nonempty intersection, then J' ≤ J.

          If π is a partition of I, then there exists a finite set s of hyperplanes such that splitMany I s ≤ π.

          For every prepartition π of I there exists a prepartition that covers exactly I \ π.iUnion.

          If π is a prepartition of I, then π.compl is a prepartition of I such that π.compl.iUnion = I \ π.iUnion.

          Equations
          Instances For