Induction on subboxes #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove (see
box_integral.tagged_partition.exists_is_Henstock_is_subordinate_homothetic) that for every box I
in ℝⁿ and a function r : ℝⁿ → ℝ positive on I there exists a tagged partition π of I such
that
- πis a Henstock partition;
- πis subordinate to- r;
- each box in πis homothetic toIwith coefficient of the form1 / 2 ^ n.
Later we will use this lemma to prove that the Henstock filter is nontrivial, hence the Henstock integral is well-defined.
Tags #
partition, tagged partition, Henstock integral
Split a box in ℝⁿ into 2 ^ n boxes by hyperplanes passing through its center.
Equations
Let p be a predicate on box ι, let I be a box. Suppose that the following two properties
hold true.
- Consider a smaller box J ≤ I. The hyperplanes passing through the center ofJsplit it into2 ^ nboxes. Ifpholds true on each of these boxes, then it true onJ.
- For each zin the closed boxI.Iccthere exists a neighborhoodUofzwithinI.Iccsuch that for every boxJ ≤ Isuch thatz ∈ J.Icc ⊆ U, ifJis homothetic toIwith a coefficient of the form1 / 2 ^ m, thenpis true onJ.
Then p I is true. See also box_integral.box.subbox_induction_on' for a version using
box_integral.box.split_center_box instead of box_integral.prepartition.split_center.
Given a box I in ℝⁿ and a function r : ℝⁿ → (0, ∞), there exists a tagged partition π of
I such that
- πis a Henstock partition;
- πis subordinate to- r;
- each box in πis homothetic toIwith coefficient of the form1 / 2 ^ m.
This lemma implies that the Henstock filter is nontrivial, hence the Henstock integral is well-defined.
Given a box I in ℝⁿ, a function r : ℝⁿ → (0, ∞), and a prepartition π of I, there
exists a tagged prepartition π' of I such that
- each box of π'is included in some box ofπ;
- π'is a Henstock partition;
- π'is subordinate to- r;
- π'covers exactly the same part of- Ias- π;
- the distortion of π'is equal to the distortion ofπ.
Given a prepartition π of a box I and a function r : ℝⁿ → (0, ∞), π.to_subordinate r
is a tagged partition π' such that
- each box of π'is included in some box ofπ;
- π'is a Henstock partition;
- π'is subordinate to- r;
- π'covers exactly the same part of- Ias- π;
- the distortion of π'is equal to the distortion ofπ.
Equations
- π.to_subordinate r = _.some
Given a tagged prepartition π₁, a prepartition π₂ that covers exactly I \ π₁.Union, and
a function r : ℝⁿ → (0, ∞), returns the union of π₁ and π₂.to_subordinate r. This partition
π has the following properties:
- πis a partition, i.e. it covers the whole- I;
- π₁.boxes ⊆ π.boxes;
- π.tag J = π₁.tag Jwhenever- J ∈ π₁;
- πis Henstock outside of- π₁:- π.tag J ∈ J.Iccwhenever- J ∈ π,- J ∉ π₁;
- πis subordinate to- routside of- π₁;
- the distortion of πis equal to the maximum of the distortions ofπ₁andπ₂.
Equations
- π₁.union_compl_to_subordinate π₂ hU r = π₁.disj_union (π₂.to_subordinate r) _