mathlib3 documentation

analysis.box_integral.partition.split

Split a box along one or more hyperplanes #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Main definitions #

A hyperplane {x : ι → ℝ | x i = a} splits a rectangular box I : box_integral.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 box_integral.box.

We introduce the following definitions.

Main results #

The main result box_integral.prepartition.exists_Union_eq_diff says that any prepartition π of I admits a prepartition π' of I that covers exactly I \ π.Union. One of these prepartitions is available as box_integral.prepartition.compl.

Tags #

rectangular box, partition, hyperplane

noncomputable def box_integral.box.split_lower {ι : Type u_1} (I : box_integral.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. box_integral.box.split_lower 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 with_bot (box_integral.box ι).

Equations
@[simp]
theorem box_integral.box.coe_split_lower {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
(I.split_lower i x) = I {y : ι | y i x}
theorem box_integral.box.split_lower_le {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
@[simp]
theorem box_integral.box.split_lower_eq_bot {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
@[simp]
theorem box_integral.box.split_lower_eq_self {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
I.split_lower i x = I I.upper i x
theorem box_integral.box.split_lower_def {ι : Type u_1} {I : box_integral.box ι} [decidable_eq ι] {i : ι} {x : } (h : x set.Ioo (I.lower i) (I.upper i)) (h' : ( (j : ι), I.lower j < function.update I.upper i x j) := _) :
noncomputable def box_integral.box.split_upper {ι : Type u_1} (I : box_integral.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. box_integral.box.split_upper 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 with_bot (box_integral.box ι).

Equations
@[simp]
theorem box_integral.box.coe_split_upper {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
(I.split_upper i x) = I {y : ι | x < y i}
theorem box_integral.box.split_upper_le {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
@[simp]
theorem box_integral.box.split_upper_eq_bot {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
@[simp]
theorem box_integral.box.split_upper_eq_self {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } :
I.split_upper i x = I x I.lower i
theorem box_integral.box.split_upper_def {ι : Type u_1} {I : box_integral.box ι} [decidable_eq ι] {i : ι} {x : } (h : x set.Ioo (I.lower i) (I.upper i)) (h' : ( (j : ι), function.update I.lower i x j < I.upper j) := _) :
theorem box_integral.box.split_lower_ne_split_upper {ι : Type u_1} (I : box_integral.box ι) (i : ι) (x : ) :
noncomputable def box_integral.prepartition.split {ι : Type u_1} (I : box_integral.box ι) (i : ι) (x : ) :

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
@[simp]
theorem box_integral.prepartition.mem_split_iff' {ι : Type u_1} {I J : box_integral.box ι} {i : ι} {x : } :
J box_integral.prepartition.split I i x J = I {y : ι | y i x} J = I {y : ι | x < y i}
@[simp]
theorem box_integral.prepartition.sum_split_boxes {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] (I : box_integral.box ι) (i : ι) (x : ) (f : box_integral.box ι M) :
theorem box_integral.prepartition.split_of_not_mem_Ioo {ι : Type u_1} {I : box_integral.box ι} {i : ι} {x : } (h : x set.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 box_integral.prepartition.coe_eq_of_mem_split_of_mem_le {ι : Type u_1} {I J : box_integral.box ι} {i : ι} {x : } {y : ι } (h₁ : J box_integral.prepartition.split I i x) (h₂ : y J) (h₃ : y i x) :
J = I {y : ι | y i x}
theorem box_integral.prepartition.coe_eq_of_mem_split_of_lt_mem {ι : Type u_1} {I J : box_integral.box ι} {i : ι} {x : } {y : ι } (h₁ : J box_integral.prepartition.split I i x) (h₂ : y J) (h₃ : x < y i) :
J = I {y : ι | x < y i}
noncomputable def box_integral.prepartition.split_many {ι : Type u_1} (I : box_integral.box ι) (s : finset × )) :

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

Equations
theorem box_integral.prepartition.not_disjoint_imp_le_of_subset_of_mem_split_many {ι : Type u_1} {I J Js : box_integral.box ι} {s : finset × )} (H : (i : ι), {(i, J.lower i), (i, J.upper i)} s) (HJs : Js box_integral.prepartition.split_many 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.

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 split_many I s ≤ π.

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

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

Equations
theorem box_integral.prepartition.compl_congr {ι : Type u_1} {I : box_integral.box ι} [finite ι] {π₁ π₂ : box_integral.prepartition I} (h : π₁.Union = π₂.Union) :
π₁.compl = π₂.compl

Since the definition of box_integral.prepartition.compl uses Exists.some, the result depends only on π.Union.

@[simp]