Filters used in box-based integrals #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
First we define a structure box_integral.integration_params
. This structure will be used as an
argument in the definition of box_integral.integral
in order to use the same definition for a few
well-known definitions of integrals based on partitions of a rectangular box into subboxes (Riemann
integral, Henstock-Kurzweil integral, and McShane integral).
This structure holds three boolean values (see below), and encodes eight different sets of
parameters; only four of these values are used somewhere in mathlib
. Three of them correspond to
the integration theories listed above, and one is a generalization of the one-dimensional
Henstock-Kurzweil integral such that the divergence theorem works without additional integrability
assumptions.
Finally, for each set of parameters l : box_integral.integration_params
and a rectangular box
I : box_integral.box ι
, we define several filter
s that will be used either in the definition of
the corresponding integral, or in the proofs of its properties. We equip
box_integral.integration_params
with a bounded_order
structure such that larger
integration_params
produce larger filters.
Main definitions #
Integration parameters #
The structure box_integral.integration_params
has 3 boolean fields with the following meaning:
-
bRiemann
: the valuett
means that the filter corresponds to a Riemann-style integral, i.e. in the definition of integrability we require a constant upper estimater
on the size of boxes of a tagged partition; the valueff
means that the estimate may depend on the position of the tag. -
bHenstock
: the valuett
means that we require that each tag belongs to its own closed box; the valueff
means that we only require that tags belong to the ambient box. -
bDistortion
: the valuett
means thatr
can depend on the maximal ratio of sides of the same box of a partition. Presence of this case make quite a few proofs harder but we can prove the divergence theorem only for the filterbox_integral.integration_params.GP = ⊥ = {bRiemann := ff, bHenstock := tt, bDistortion := tt}
.
Well-known sets of parameters #
Out of eight possible values of box_integral.integration_params
, the following four are used in
the library.
-
box_integral.integration_params.Riemann
(bRiemann = tt
,bHenstock = tt
,bDistortion = ff
): this value corresponds to the Riemann integral; in the corresponding filter, we require that the diameters of all boxesJ
of a tagged partition are bounded from above by a constant upper estimate that may not depend on the geometry ofJ
, and each tag belongs to the corresponding closed box. -
box_integral.integration_params.Henstock
(bRiemann = ff
,bHenstock = tt
,bDistortion = ff
): this value corresponds to the most natural generalization of Henstock-Kurzweil integral to higher dimension; the only (but important!) difference between this theory and Riemann integral is that instead of a constant upper estimate on the size of all boxes of a partition, we require that the partition is subordinate to a possibly discontinuous functionr : (ι → ℝ) → {x : ℝ | 0 < x}
, i.e. each boxJ
is included in a closed ball with centerπ.tag J
and radiusr J
. -
box_integral.integration_params.McShane
(bRiemann = ff
,bHenstock = ff
,bDistortion = ff
): this value corresponds to the McShane integral; the only difference with the Henstock integral is that we allow tags to be outside of their boxes; the tags still have to be in the ambient closed box, and the partition still has to be subordinate to a function. -
box_integral.integration_params.GP = ⊥
(bRiemann = ff
,bHenstock = tt
,bDistortion = tt
): this is the least integration theory in our list, i.e., all functions integrable in any other theory is integrable in this one as well. This is a non-standard generalization of the Henstock-Kurzweil integral to higher dimension. In dimension one, it generates the same filter asHenstock
. In higher dimension, this generalization defines an integration theory such that the divergence of any Fréchet differentiable functionf
is integrable, and its integral is equal to the sum of integrals off
over the faces of the box, taken with appropriate signs.A function
f
isGP
-integrable if for anyε > 0
andc : ℝ≥0
there existsr : (ι → ℝ) → {x : ℝ | 0 < x}
such that for any tagged partitionπ
subordinate tor
, if each tag belongs to the corresponding closed box and for each boxJ ∈ π
, the maximal ratio of its sides is less than or equal toc
, then the integral sum off
overπ
isε
-close to the integral.
Filters and predicates on tagged_prepartition I
#
For each value of integration_params
and a rectangular box I
, we define a few filters on
tagged_prepartition I
. First, we define a predicate
structure box_integral.integration_params.mem_base_set (l : box_integral.integration_params)
(I : box_integral.box ι) (c : ℝ≥0) (r : (ι → ℝ) → Ioi (0 : ℝ))
(π : box_integral.tagged_prepartition I) : Prop :=
This predicate says that
- if
l.bHenstock
, thenπ
is a Henstock prepartition, i.e. each tag belongs to the corresponding closed box; π
is subordinate tor
;- if
l.bDistortion
, then the distortion of each box inπ
is less than or equal toc
; - if
l.bDistortion
, then there exists a prepartitionπ'
with distortion≤ c
that covers exactlyI \ π.Union
.
The last condition is always true for c > 1
, see TODO section for more details.
Then we define a predicate box_integral.integration_params.r_cond
on functions
r : (ι → ℝ) → {x : ℝ | 0 < x}
. If l.bRiemann
, then this predicate requires r
to be a constant
function, otherwise it imposes no restrictions on r
. We introduce this definition to prove a few
dot-notation lemmas: e.g., box_integral.integration_params.r_cond.min
says that the pointwise
minimum of two functions that satisfy this condition satisfies this condition as well.
Then we define four filters on box_integral.tagged_prepartition I
.
-
box_integral.integration_params.to_filter_distortion
: an auxiliary filter that takes parameters(l : box_integral.integration_params) (I : box_integral.box ι) (c : ℝ≥0)
and returns the filter generated by all sets{π | mem_base_set l I c r π}
, wherer
is a function satisfying the predicatebox_integral.integration_params.r_cond l
; -
box_integral.integration_params.to_filter l I
: the supremum ofl.to_filter_distortion I c
over allc : ℝ≥0
; -
box_integral.integration_params.to_filter_distortion_Union l I c π₀
, whereπ₀
is a prepartition ofI
: the infimum ofl.to_filter_distortion I c
and the principal filter generated by{π | π.Union = π₀.Union}
; -
box_integral.integration_params.to_filter_Union l I π₀
: the supremum ofl.to_filter_distortion_Union l I c π₀
over allc : ℝ≥0
. This is the filter (in the caseπ₀ = ⊤
is the one-box partition ofI
) used in the definition of the integral of a function over a box.
Implementation details #
-
Later we define the integral of a function over a rectangular box as the limit (if it exists) of the integral sums along
box_integral.integration_params.to_filter_Union l I ⊤
. While it is possible to define the integral with a general filter onbox_integral.tagged_prepartition I
as a parameter, many lemmas (e.g., Sacks-Henstock lemma and most results about integrability of functions) require the filter to have a predictable structure. So, instead of adding assumptions about the filter here and there, we define this auxiliary type that can encode all integration theories we need in practice. -
While the definition of the integral only uses the filter
box_integral.integration_params.to_filter_Union l I ⊤
and partitions of a box, some lemmas (e.g., the Henstock-Sacks lemmas) are best formulated in terms of the predicatemem_base_set
and other filters defined above. -
We use
bool
instead ofProp
for the fields ofintegration_params
in order to have decidable equality and inequalities.
TODO #
Currently, box_integral.integration_params.mem_base_set
explicitly requires that there exists a
partition of the complement I \ π.Union
with distortion ≤ c
. For c > 1
, this condition is
always true but the proof of this fact requires more API about
box_integral.prepartition.split_many
. We should formalize this fact, then either require c > 1
everywhere, or replace ≤ c
with < c
so that we automatically get c > 1
for a non-trivial
prepartition (and consider the special case π = ⊥
separately if needed).
Tags #
integral, rectangular box, partition, filter
An integration_params
is a structure holding 3 boolean values used to define a filter to be
used in the definition of a box-integrable function.
-
bRiemann
: the valuett
means that the filter corresponds to a Riemann-style integral, i.e. in the definition of integrability we require a constant upper estimater
on the size of boxes of a tagged partition; the valueff
means that the estimate may depend on the position of the tag. -
bHenstock
: the valuett
means that we require that each tag belongs to its own closed box; the valueff
means that we only require that tags belong to the ambient box. -
bDistortion
: the valuett
means thatr
can depend on the maximal ratio of sides of the same box of a partition. Presence of this case makes quite a few proofs harder but we can prove the divergence theorem only for the filterbox_integral.integration_params.GP = ⊥ = {bRiemann := ff, bHenstock := tt, bDistortion := tt}
.
Instances for box_integral.integration_params
- box_integral.integration_params.has_sizeof_inst
- box_integral.integration_params.partial_order
- box_integral.integration_params.bounded_order
- box_integral.integration_params.inhabited
Auxiliary equivalence with a product type used to lift an order.
Equations
- box_integral.integration_params.equiv_prod = {to_fun := λ (l : box_integral.integration_params), (l.bRiemann, ⇑order_dual.to_dual l.bHenstock, ⇑order_dual.to_dual l.bDistortion), inv_fun := λ (l : bool × boolᵒᵈ × boolᵒᵈ), {bRiemann := l.fst, bHenstock := ⇑order_dual.of_dual l.snd.fst, bDistortion := ⇑order_dual.of_dual l.snd.snd}, left_inv := box_integral.integration_params.equiv_prod._proof_1, right_inv := box_integral.integration_params.equiv_prod._proof_2}
Equations
- box_integral.integration_params.partial_order = partial_order.lift ⇑box_integral.integration_params.equiv_prod box_integral.integration_params.partial_order._proof_1
Auxiliary order_iso
with a product type used to lift a bounded_order
structure.
Equations
- box_integral.integration_params.iso_prod = {to_equiv := box_integral.integration_params.equiv_prod, map_rel_iff' := box_integral.integration_params.iso_prod._proof_1}
The value
box_integral.integration_params.GP = ⊥
(bRiemann = ff
, bHenstock = tt
, bDistortion = tt
)
corresponds to a generalization of the Henstock integral such that the Divergence theorem holds true
without additional integrability assumptions, see the module docstring for details.
Equations
Equations
Equations
- box_integral.integration_params.decidable_eq = λ (x y : box_integral.integration_params), decidable_of_iff (x.bRiemann = y.bRiemann ∧ x.bHenstock = y.bHenstock ∧ x.bDistortion = y.bDistortion) _
The box_integral.integration_params
corresponding to the Riemann integral. In the
corresponding filter, we require that the diameters of all boxes J
of a tagged partition are
bounded from above by a constant upper estimate that may not depend on the geometry of J
, and each
tag belongs to the corresponding closed box.
Equations
The box_integral.integration_params
corresponding to the Henstock-Kurzweil integral. In the
corresponding filter, we require that the tagged partition is subordinate to a (possibly,
discontinuous) positive function r
and each tag belongs to the corresponding closed box.
Equations
The box_integral.integration_params
corresponding to the McShane integral. In the
corresponding filter, we require that the tagged partition is subordinate to a (possibly,
discontinuous) positive function r
; the tags may be outside of the corresponding closed box
(but still inside the ambient closed box I.Icc
).
Equations
The box_integral.integration_params
corresponding to the generalized Perron integral. In the
corresponding filter, we require that the tagged partition is subordinate to a (possibly,
discontinuous) positive function r
and each tag belongs to the corresponding closed box. We also
require an upper estimate on the distortion of all boxes of the partition.
Equations
- is_subordinate : π.is_subordinate r
- is_Henstock : ↥(l.bHenstock) → π.is_Henstock
- distortion_le : ↥(l.bDistortion) → π.distortion ≤ c
- exists_compl : ↥(l.bDistortion) → (∃ (π' : box_integral.prepartition I), π'.Union = ↑I \ π.Union ∧ π'.distortion ≤ c)
The predicate corresponding to a base set of the filter defined by an
integration_params
. It says that
- if
l.bHenstock
, thenπ
is a Henstock prepartition, i.e. each tag belongs to the corresponding closed box; π
is subordinate tor
;- if
l.bDistortion
, then the distortion of each box inπ
is less than or equal toc
; - if
l.bDistortion
, then there exists a prepartitionπ'
with distortion≤ c
that covers exactlyI \ π.Union
.
The last condition is automatically verified for partitions, and is used in the proof of the Sacks-Henstock inequality to compare two prepartitions covering the same part of the box.
It is also automatically satisfied for any c > 1
, see TODO section of the module docstring for
details.
A set s : set (tagged_prepartition I)
belongs to l.to_filter_distortion I c
if there exists
a function r : ℝⁿ → (0, ∞)
(or a constant r
if l.bRiemann = tt
) such that s
contains each
prepartition π
such that l.mem_base_set I c r π
.
Equations
- l.to_filter_distortion I c = ⨅ (r : (ι → ℝ) → ↥(set.Ioi 0)) (hr : l.r_cond r), filter.principal {π : box_integral.tagged_prepartition I | l.mem_base_set I c r π}
Instances for box_integral.integration_params.to_filter_distortion
A set s : set (tagged_prepartition I)
belongs to l.to_filter I
if for any c : ℝ≥0
there
exists a function r : ℝⁿ → (0, ∞)
(or a constant r
if l.bRiemann = tt
) such that
s
contains each prepartition π
such that l.mem_base_set I c r π
.
Instances for box_integral.integration_params.to_filter
A set s : set (tagged_prepartition I)
belongs to l.to_filter_distortion_Union I c π₀
if
there exists a function r : ℝⁿ → (0, ∞)
(or a constant r
if l.bRiemann = tt
) such that s
contains each prepartition π
such that l.mem_base_set I c r π
and π.Union = π₀.Union
.
Equations
- l.to_filter_distortion_Union I c π₀ = l.to_filter_distortion I c ⊓ filter.principal {π : box_integral.tagged_prepartition I | π.Union = π₀.Union}
Instances for box_integral.integration_params.to_filter_distortion_Union
A set s : set (tagged_prepartition I)
belongs to l.to_filter_Union I π₀
if for any c : ℝ≥0
there exists a function r : ℝⁿ → (0, ∞)
(or a constant r
if l.bRiemann = tt
) such that s
contains each prepartition π
such that l.mem_base_set I c r π
and π.Union = π₀.Union
.
Equations
- l.to_filter_Union I π₀ = ⨆ (c : nnreal), l.to_filter_distortion_Union I c π₀