Skip to content

Commit

Permalink
Update Mathlib/MeasureTheory/Integral/IntervalIntegral.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Jon Eugster <eugster.jon@gmail.com>
  • Loading branch information
kebekus and joneugster authored Jan 14, 2025
1 parent 1f946ff commit f821b70
Showing 1 changed file with 3 additions and 5 deletions.
8 changes: 3 additions & 5 deletions Mathlib/MeasureTheory/Integral/IntervalIntegral.lean
Original file line number Diff line number Diff line change
Expand Up @@ -385,11 +385,9 @@ of the form `0..x` if it is interval integrable (with respect to the volume meas
interval of the form `0..x`, for positive `x`.
See `intervalIntegrable_of_even` for a stronger result.-/
lemma intervalIntegrable_of_even₀
(h₁f : ∀ x, f x = f (-x))
(h₂f : ∀ x, 0 < x → IntervalIntegrable f volume 0 x)
(t : ℝ) :
IntervalIntegrable f volume 0 t := by
lemma intervalIntegrable_of_even₀ (h₁f : ∀ x, f x = f (-x))
(h₂f : ∀ x, 0 < x → IntervalIntegrable f volume 0 x) (t : ℝ) :
IntervalIntegrable f volume 0 t := by
rcases lt_trichotomy t 0 with h | h | h
· rw [IntervalIntegrable.iff_comp_neg]
conv => arg 1; intro t; rw [← h₁f]
Expand Down

0 comments on commit f821b70

Please sign in to comment.