Update Basic.lean
Some checks failed
Lean Action CI / build (push) Has been cancelled

This commit is contained in:
Stefan Kebekus
2025-12-13 07:15:12 +01:00
parent 6de85b8db6
commit 6ec755312b

View File

@@ -1,8 +1,15 @@
import Mathlib
variable
{E : Type*} [NormedAddCommGroup E] [NormedSpace E]
lemma MeromorphicAt.comp {x : } {f : E} {g : }
(hf : MeromorphicAt f (g x)) (hg : AnalyticAt g x) : MeromorphicAt (f g) x := by
theorem intervalIntegrable_iff_intervalIntegrable_smul
{E : Type*} [NormedAddCommGroup E]
{a b : } {μ : MeasureTheory.Measure }
{R : Type*} [NormedAddCommGroup R] [SMulZeroClass R E] [IsBoundedSMul R E]
{f : E} {r : R} (hr : r 0) :
IntervalIntegrable f μ a b IntervalIntegrable (r f) μ a b := by
sorry
theorem IntervalIntegrable.abs'
{a b : } {μ : MeasureTheory.Measure } {f : } (hf : Measurable f) :
IntervalIntegrable f μ a b IntervalIntegrable (fun x => |f x|) μ a b := by
sorry