Skip to content

Commit 4f8cced

Browse files
feat: add Integrable.of_integral_ne_zero (#10430)
1 parent b005724 commit 4f8cced

File tree

1 file changed

+5
-2
lines changed

1 file changed

+5
-2
lines changed

Mathlib/MeasureTheory/Integral/Bochner.lean

Lines changed: 5 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -839,6 +839,9 @@ theorem integral_undef {f : α → G} (h : ¬Integrable f μ) : ∫ a, f a ∂μ
839839
· simp [integral, hG]
840840
#align measure_theory.integral_undef MeasureTheory.integral_undef
841841

842+
theorem Integrable.of_integral_ne_zero {f : α → G} (h : ∫ a, f a ∂μ ≠ 0) : Integrable f μ :=
843+
Not.imp_symm integral_undef h
844+
842845
theorem integral_non_aestronglyMeasurable {f : α → G} (h : ¬AEStronglyMeasurable f μ) :
843846
∫ a, f a ∂μ = 0 :=
844847
integral_undef <| not_and_of_not_left _ h
@@ -861,8 +864,8 @@ theorem integral_zero' : integral μ (0 : α → G) = 0 :=
861864

862865
variable {α G}
863866

864-
theorem integrable_of_integral_eq_one {f : α → ℝ} (h : ∫ x, f x ∂μ = 1) : Integrable f μ := by
865-
contrapose h; rw [integral_undef h]; exact zero_ne_one
867+
theorem integrable_of_integral_eq_one {f : α → ℝ} (h : ∫ x, f x ∂μ = 1) : Integrable f μ :=
868+
.of_integral_ne_zero <| h ▸ one_ne_zero
866869
#align measure_theory.integrable_of_integral_eq_one MeasureTheory.integrable_of_integral_eq_one
867870

868871
theorem integral_add {f g : α → G} (hf : Integrable f μ) (hg : Integrable g μ) :

0 commit comments

Comments
 (0)