Skip to content

Commit

Permalink
rclike
Browse files Browse the repository at this point in the history
  • Loading branch information
arulandu committed Oct 3, 2024
1 parent 1ab8987 commit f67bf07
Showing 1 changed file with 10 additions and 8 deletions.
18 changes: 10 additions & 8 deletions Mathlib/MeasureTheory/Integral/IntegrableOn.lean
Original file line number Diff line number Diff line change
Expand Up @@ -697,22 +697,24 @@ theorem integrableOn_Iic_iff_integrableOn_Iio :
end PartialOrder

namespace MeasureTheory
variable {X : Type*} [MeasurableSpace X] {μ : Measure X} {s : Set X}
variable {X : Type*} [MeasurableSpace X] {𝕜 : Type*} [RCLike 𝕜] {μ : Measure X} {s : Set X}
theorem IntegrableOn.iff_ofReal {f : X → ℝ} :
IntegrableOn f s μ ↔ IntegrableOn (fun x ↦ (f x : ℂ)) s μ :=
MeasureTheory.Integrable.iff_ofReal

theorem IntegrableOn.ofReal {f : X → ℝ} (hf : IntegrableOn f s μ) :
IntegrableOn (fun x => (f x : ℂ)) s μ := IntegrableOn.iff_ofReal.1 hf
IntegrableOn (fun x => (f x : 𝕜)) s μ := by
rw [IntegrableOn, ← memℒp_one_iff_integrable] at hf ⊢
exact hf.ofReal

theorem IntegrableOn.re_im_iff {f : X → } :
IntegrableOn (fun x => (f x).re) s μ ∧ IntegrableOn (fun x => (f x).im) s μ ↔
theorem IntegrableOn.re_im_iff {f : X → 𝕜} :
IntegrableOn (fun x => RCLike.re (f x)) s μ ∧ IntegrableOn (fun x => RCLike.im (f x)) s μ ↔
IntegrableOn f s μ := Integrable.re_im_iff (f := f)

theorem IntegrableOn.re {f : X → } (hf : IntegrableOn f s μ) :
IntegrableOn (fun x => (f x).re) s μ := (IntegrableOn.re_im_iff.2 hf).left
theorem IntegrableOn.re {f : X → 𝕜} (hf : IntegrableOn f s μ) :
IntegrableOn (fun x => RCLike.re (f x)) s μ := (IntegrableOn.re_im_iff.2 hf).left

theorem IntegrableOn.im {f : X → } (hf : IntegrableOn f s μ) :
IntegrableOn (fun x => (f x).im) s μ := (IntegrableOn.re_im_iff.2 hf).right
theorem IntegrableOn.im {f : X → 𝕜} (hf : IntegrableOn f s μ) :
IntegrableOn (fun x => RCLike.im (f x)) s μ := (IntegrableOn.re_im_iff.2 hf).right

end MeasureTheory

0 comments on commit f67bf07

Please sign in to comment.