mathlib3 documentation

analysis.box_integral.partition.additive

Box additive functions #

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

We say that a function f : box ι → M from boxes in ℝⁿ to a commutative additive monoid M is box additive on subboxes of I₀ : with_top (box ι) if for any box J, ↑J ≤ I₀, and a partition π of J, f J = ∑ J' in π.boxes, f J'. We use I₀ : with_top (box ι) instead of I₀ : box ι to use the same definition for functions box additive on subboxes of a box and for functions box additive on all boxes.

Examples of box-additive functions include the measure of a box and the integral of a fixed integrable function over a box.

In this file we define box-additive functions and prove that a function such that f J = f (J ∩ {x | x i < y}) + f (J ∩ {x | y ≤ x i}) is box-additive.

Tags #

rectangular box, additive function

structure box_integral.box_additive_map (ι : Type u_3) (M : Type u_4) [add_comm_monoid M] (I : with_top (box_integral.box ι)) :
Type (max u_3 u_4)

A function on box ι is called box additive if for every box J and a partition π of J we have f J = ∑ Ji in π.boxes, f Ji. A function is called box additive on subboxes of I : box ι if the same property holds for J ≤ I. We formalize these two notions in the same definition using I : with_bot (box ι): the value I = ⊤ corresponds to functions box additive on the whole space.

Instances for box_integral.box_additive_map
@[simp]
theorem box_integral.box_additive_map.coe_mk {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] {I₀ : with_top (box_integral.box ι)} (f : box_integral.box ι M) (h : (J : box_integral.box ι), J I₀ (π : box_integral.prepartition J), π.is_partition π.boxes.sum (λ (Ji : box_integral.box ι), f Ji) = f J) :
@[simp]
theorem box_integral.box_additive_map.coe_inj {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] {I₀ : with_top (box_integral.box ι)} {f g : box_integral.box_additive_map ι M I₀} :
f = g f = g
theorem box_integral.box_additive_map.sum_partition_boxes {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] {I₀ : with_top (box_integral.box ι)} {I : box_integral.box ι} (f : box_integral.box_additive_map ι M I₀) (hI : I I₀) {π : box_integral.prepartition I} (h : π.is_partition) :
π.boxes.sum (λ (J : box_integral.box ι), f J) = f I
@[simp]
@[protected, instance]
Equations
@[protected, instance]
Equations
@[simp]
theorem box_integral.box_additive_map.map_split_add {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] {I₀ : with_top (box_integral.box ι)} {I : box_integral.box ι} (f : box_integral.box_additive_map ι M I₀) (hI : I I₀) (i : ι) (x : ) :
@[simp]
theorem box_integral.box_additive_map.restrict_apply {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] {I₀ : with_top (box_integral.box ι)} (f : box_integral.box_additive_map ι M I₀) (I : with_top (box_integral.box ι)) (hI : I I₀) (ᾰ : box_integral.box ι) :
(f.restrict I hI) = f ᾰ

If f is box-additive on subboxes of I₀, then it is box-additive on subboxes of any I ≤ I₀.

Equations
def box_integral.box_additive_map.of_map_split_add {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] [fintype ι] (f : box_integral.box ι M) (I₀ : with_top (box_integral.box ι)) (hf : (I : box_integral.box ι), I I₀ {i : ι} {x : }, x set.Ioo (I.lower i) (I.upper i) option.elim 0 f (I.split_lower i x) + option.elim 0 f (I.split_upper i x) = f I) :

If f : box ι → M is box additive on partitions of the form split I i x, then it is box additive.

Equations
def box_integral.box_additive_map.map {ι : Type u_1} {M : Type u_2} {N : Type u_3} [add_comm_monoid M] [add_comm_monoid N] {I₀ : with_top (box_integral.box ι)} (f : box_integral.box_additive_map ι M I₀) (g : M →+ N) :

If g : M → N is an additive map and f is a box additive map, then g ∘ f is a box additive map.

Equations
@[simp]
theorem box_integral.box_additive_map.map_apply {ι : Type u_1} {M : Type u_2} {N : Type u_3} [add_comm_monoid M] [add_comm_monoid N] {I₀ : with_top (box_integral.box ι)} (f : box_integral.box_additive_map ι M I₀) (g : M →+ N) :
(f.map g) = g f
theorem box_integral.box_additive_map.sum_boxes_congr {ι : Type u_1} {M : Type u_2} [add_comm_monoid M] {I₀ : with_top (box_integral.box ι)} {I : box_integral.box ι} [finite ι] (f : box_integral.box_additive_map ι M I₀) (hI : I I₀) {π₁ π₂ : box_integral.prepartition I} (h : π₁.Union = π₂.Union) :
π₁.boxes.sum (λ (J : box_integral.box ι), f J) = π₂.boxes.sum (λ (J : box_integral.box ι), f J)

If f is a box additive function on subboxes of I and π₁, π₂ are two prepartitions of I that cover the same part of I, then ∑ J in π₁.boxes, f J = ∑ J in π₂.boxes, f J.

If f is a box-additive map, then so is the map sending I to the scalar multiplication by f I as a continuous linear map from E to itself.

Equations
@[simp]
@[simp]
theorem box_integral.box_additive_map.upper_sub_lower_apply {n : } {G : Type u} [add_comm_group G] (I₀ : box_integral.box (fin (n + 1))) (i : fin (n + 1)) (f : box_integral.box (fin n) G) (fb : (set.Icc (I₀.lower i) (I₀.upper i)) box_integral.box_additive_map (fin n) G (I₀.face i)) (hf : (x : ) (hx : x set.Icc (I₀.lower i) (I₀.upper i)) (J : box_integral.box (fin n)), f x J = (fb x, hx⟩) J) (J : box_integral.box (fin (n + 1))) :
(box_integral.box_additive_map.upper_sub_lower I₀ i f fb hf) J = f (J.upper i) (J.face i) - f (J.lower i) (J.face i)
def box_integral.box_additive_map.upper_sub_lower {n : } {G : Type u} [add_comm_group G] (I₀ : box_integral.box (fin (n + 1))) (i : fin (n + 1)) (f : box_integral.box (fin n) G) (fb : (set.Icc (I₀.lower i) (I₀.upper i)) box_integral.box_additive_map (fin n) G (I₀.face i)) (hf : (x : ) (hx : x set.Icc (I₀.lower i) (I₀.upper i)) (J : box_integral.box (fin n)), f x J = (fb x, hx⟩) J) :

Given a box I₀ in ℝⁿ⁺¹, f x : box (fin n) → G is a family of functions indexed by a real x and for x ∈ [I₀.lower i, I₀.upper i], f x is box-additive on subboxes of the i-th face of I₀, then λ J, f (J.upper i) (J.face i) - f (J.lower i) (J.face i) is box-additive on subboxes of I₀.

Equations