mathlib3 documentation

measure_theory.function.locally_integrable

Locally integrable functions #

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

A function is called locally integrable (measure_theory.locally_integrable) if it is integrable on a neighborhood of every point. More generally, it is locally integrable on s if it is locally integrable on a neighbourhood within s of any point of s.

This file contains properties of locally integrable functions, and integrability results on compact sets.

Main statements #

def measure_theory.locally_integrable_on {X : Type u_1} {E : Type u_3} [measurable_space X] [topological_space X] [normed_add_comm_group E] (f : X E) (s : set X) (μ : measure_theory.measure X . "volume_tac") :
Prop

A function f : X → E is locally integrable on s, for s ⊆ X, if for every x ∈ s there is a neighbourhood of x within s on which f is integrable. (Note this is, in general, strictly weaker than local integrability with respect to μ.restrict s.)

Equations

If a function is locally integrable on a compact set, then it is integrable on that set.

If s is either open, or closed, then f is locally integrable on s iff it is integrable on every compact subset contained in s.

def measure_theory.locally_integrable {X : Type u_1} {E : Type u_3} [measurable_space X] [topological_space X] [normed_add_comm_group E] (f : X E) (μ : measure_theory.measure X . "volume_tac") :
Prop

A function f : X → E is locally integrable if it is integrable on a neighborhood of every point. In particular, it is integrable on all compact sets, see locally_integrable.integrable_on_is_compact.

Equations

If f is locally integrable with respect to μ.restrict s, it is locally integrable on s. (See locally_integrable_on_iff_locally_integrable_restrict for an iff statement when s is closed.)

If s is closed, being locally integrable on s wrt μ is equivalent to being locally integrable with respect to μ.restrict s. For the one-way implication without assuming s closed, see locally_integrable_on_of_locally_integrable_restrict.

If a function is locally integrable, then it is integrable on any compact set.

If a function is locally integrable, then it is integrable on an open neighborhood of any compact set.

A continuous function f is locally integrable with respect to any locally finite measure.

A function f continuous on a set K is locally integrable on this set with respect to any locally finite measure.

A function f continuous on a compact set K is integrable on this set with respect to any locally finite measure.

A continuous function with compact support is integrable on the whole space.

theorem measure_theory.integrable_on.continuous_on_smul {X : Type u_1} {E : Type u_3} [measurable_space X] [topological_space X] [normed_add_comm_group E] {μ : measure_theory.measure X} [opens_measurable_space X] {K : set X} {𝕜 : Type u_5} [normed_field 𝕜] [normed_space 𝕜 E] [t2_space X] [second_countable_topology_either X 𝕜] {g : X E} (hg : measure_theory.integrable_on g K μ) {f : X 𝕜} (hf : continuous_on f K) (hK : is_compact K) :
measure_theory.integrable_on (λ (x : X), f x g x) K μ