MeasureTheory.MeasureSpace.Lebesgue

このファイルでは単関数の積分の定義を行います.

コード元 MeasureTheory.MeasurableSpace.SimpleFunc

/-- A function `f` from a measurable space to any type is called *simple*,
if every preimage `f ⁻¹' {x}` is measurable, and the range is finite. This structure bundles
a function with these properties. -/
structure SimpleFunc.{u, v} (α : Type u) [MeasurableSpace α] (β : Type v) where
  toFun : α  β
  measurableSet_fiber' :  x, MeasurableSet (toFun ⁻¹' {x})
  finite_range' : (Set.range toFun).Finite

SimpleFuncは可測空間から任意の型への単関数を表します. toFunはその関数を表し, measurableSet_fiber'はその逆像が常に可測であることを示しています. finite_range'はその値域が有限であることを示しています.

local infixr:25 " →ₛ " => SimpleFunc

単関数は以上の記法で表すこともできます.

/-- Integral of a simple function whose codomain is `ℝ≥0∞`. -/
def lintegral {_m : MeasurableSpace α} (f : α →ₛ 0) (μ : Measure α) : 0 :=
   x  f.range, x * μ (f ⁻¹' {x})

lintegralは単関数の積分を定義しています. f.rangeはその値域を表します. μ (f ⁻¹' {x})はその逆像の測度を表します. x * μ (f ⁻¹' {x})はその測度に対する重み付けを行っています.