Tagged partitions #
A tagged (pre)partition is a (pre)partition π enriched with a tagged point for each box of
π. For simplicity we require that the function BoxIntegral.TaggedPrepartition.tag is defined
on all boxes J : Box ι but use its values only on boxes of the partition. Given
π : BoxIntegral.TaggedPrepartition I, we require that each BoxIntegral.TaggedPrepartition π J
belongs to BoxIntegral.Box.Icc I. If for every J ∈ π, π.tag J belongs to J.Icc, then π is
called a Henstock partition. We do not include this assumption into the definition of a tagged
(pre)partition because McShane integral is defined as a limit along tagged partitions without this
requirement.
Tags #
rectangular box, box partition
A tagged prepartition is a prepartition enriched with a tagged point for each box of the
prepartition. For simplicity we require that tag is defined for all boxes in ι → ℝ but
we will use only the values of tag on the boxes of the partition.
- boxes : Finset (BoxIntegral.Box ι)
- le_of_mem' : ∀ J ∈ self.boxes, J ≤ I
- pairwiseDisjoint : (↑self.boxes).Pairwise (Disjoint on BoxIntegral.Box.toSet)
- tag : BoxIntegral.Box ι → ι → ℝChoice of tagged point of each box in this prepartition: we extend this to a total function, on all boxes in ι → ℝ.
- tag_mem_Icc : ∀ (J : BoxIntegral.Box ι), self.tag J ∈ BoxIntegral.Box.Icc IEach tagged point belongs to I
Instances For
Each tagged point belongs to I
Equations
- BoxIntegral.TaggedPrepartition.instMembershipBox = { mem := fun (J : BoxIntegral.Box ι) (π : BoxIntegral.TaggedPrepartition I) => J ∈ π.boxes }
Union of all boxes of a tagged prepartition.
Equations
- π.iUnion = π.iUnion
Instances For
A tagged prepartition is a partition if it covers the whole box.
Equations
- π.IsPartition = π.IsPartition
Instances For
The tagged partition made of boxes of π that satisfy predicate p.
Equations
- π.filter p = { toPrepartition := π.filter p, tag := π.tag, tag_mem_Icc := ⋯ }
Instances For
Given a partition π of I : BoxIntegral.Box ι and a collection of tagged partitions
πi J of all boxes J ∈ π, returns the tagged partition of I into all the boxes of πi J
with tags coming from (πi J).tag.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a tagged partition π of I and a (not tagged) partition πi J hJ of each J ∈ π,
returns the tagged partition of I into all the boxes of all πi J hJ. The tag of a box J
is defined to be the π.tag of the box of the partition π that includes J.
Note that usually the result is not a Henstock partition.
Equations
- π.biUnionPrepartition πi = { toPrepartition := π.biUnion πi, tag := fun (J : BoxIntegral.Box ι) => π.tag (π.biUnionIndex πi J), tag_mem_Icc := ⋯ }
Instances For
Given two partitions π₁ and π₁, one of them tagged and the other is not, returns the tagged
partition with toPrepartition = π₁.toPrepartition ⊓ π₂ and tags coming from π₁.
Note that usually the result is not a Henstock partition.
Equations
- π.infPrepartition π' = π.biUnionPrepartition fun (J : BoxIntegral.Box ι) => π'.restrict J
Instances For
A tagged partition is said to be a Henstock partition if for each J ∈ π, the tag of J
belongs to J.Icc.
Instances For
In a Henstock prepartition, there are at most 2 ^ Fintype.card ι boxes with a given tag.
A tagged partition π is subordinate to r : (ι → ℝ) → ℝ if each box J ∈ π is included in
the closed ball with center π.tag J and radius r (π.tag J).
Equations
- π.IsSubordinate r = ∀ J ∈ π, BoxIntegral.Box.Icc J ⊆ Metric.closedBall (π.tag J) ↑(r (π.tag J))
Instances For
Tagged prepartition with single box and prescribed tag.
Equations
- BoxIntegral.TaggedPrepartition.single I J hJ x h = { toPrepartition := BoxIntegral.Prepartition.single I J hJ, tag := fun (x_1 : BoxIntegral.Box ι) => x, tag_mem_Icc := ⋯ }
Instances For
Equations
- BoxIntegral.TaggedPrepartition.instInhabited I = { default := BoxIntegral.TaggedPrepartition.single I I ⋯ I.upper ⋯ }
Union of two tagged prepartitions with disjoint unions of boxes.
Equations
- π₁.disjUnion π₂ h = { toPrepartition := π₁.disjUnion π₂.toPrepartition h, tag := π₁.boxes.piecewise π₁.tag π₂.tag, tag_mem_Icc := ⋯ }
Instances For
If I ≤ J, then every tagged prepartition of I is a tagged prepartition of J.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The distortion of a tagged prepartition is the maximum of distortions of its boxes.
Equations
- π.distortion = π.distortion