Complex measure #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file proves some elementary results about complex measures. In particular, we prove that
a complex measure is always in the form s + it
where s
and t
are signed measures.
The complex measure is defined to be vector measure over ℂ
, this definition can be found
in measure_theory.measure.vector_measure
and is known as measure_theory.complex_measure
.
Main definitions #
measure_theory.complex_measure.re
: obtains a signed measures
from a complex measurec
such thats i = (c i).re
for all measurable setsi
.measure_theory.complex_measure.im
: obtains a signed measures
from a complex measurec
such thats i = (c i).im
for all measurable setsi
.measure_theory.signed_measure.to_complex_measure
: given two signed measuress
andt
,s.to_complex_measure t
provides a complex measure of the forms + it
.measure_theory.complex_measure.equiv_signed_measure
: is the equivalence between the complex measures and the type of the product of the signed measures with itself.
Tags #
Complex measure
The real part of a complex measure is a signed measure.
The imaginary part of a complex measure is a signed measure.
Given s
and t
signed measures, s + it
is a complex measure
Equations
- s.to_complex_measure t = {measure_of' := λ (i : set α), {re := ⇑s i, im := ⇑t i}, empty' := _, not_measurable' := _, m_Union' := _}
The complex measures form an equivalence to the type of pairs of signed measures.
Equations
- measure_theory.complex_measure.equiv_signed_measure = {to_fun := λ (c : measure_theory.complex_measure α), (⇑measure_theory.complex_measure.re c, ⇑measure_theory.complex_measure.im c), inv_fun := λ (_x : measure_theory.signed_measure α × measure_theory.signed_measure α), measure_theory.complex_measure.equiv_signed_measure._match_1 _x, left_inv := _, right_inv := _}
- measure_theory.complex_measure.equiv_signed_measure._match_1 (s, t) = s.to_complex_measure t
The complex measures form an linear isomorphism to the type of pairs of signed measures.