File tree Expand file tree Collapse file tree 1 file changed +5
-2
lines changed
Mathlib/MeasureTheory/Integral Expand file tree Collapse file tree 1 file changed +5
-2
lines changed Original file line number Diff line number Diff line change @@ -839,6 +839,9 @@ theorem integral_undef {f : α → G} (h : ¬Integrable f μ) : ∫ a, f a ∂μ
839
839
· simp [integral, hG]
840
840
#align measure_theory.integral_undef MeasureTheory.integral_undef
841
841
842
+ theorem Integrable.of_integral_ne_zero {f : α → G} (h : ∫ a, f a ∂μ ≠ 0 ) : Integrable f μ :=
843
+ Not.imp_symm integral_undef h
844
+
842
845
theorem integral_non_aestronglyMeasurable {f : α → G} (h : ¬AEStronglyMeasurable f μ) :
843
846
∫ a, f a ∂μ = 0 :=
844
847
integral_undef <| not_and_of_not_left _ h
@@ -861,8 +864,8 @@ theorem integral_zero' : integral μ (0 : α → G) = 0 :=
861
864
862
865
variable {α G}
863
866
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
866
869
#align measure_theory.integrable_of_integral_eq_one MeasureTheory.integrable_of_integral_eq_one
867
870
868
871
theorem integral_add {f g : α → G} (hf : Integrable f μ) (hg : Integrable g μ) :
You can’t perform that action at this time.
0 commit comments