Skip to content

Commit

Permalink
chore(Analysis/SpecialFunctions/Integrals): simplify proof of interva…
Browse files Browse the repository at this point in the history
…lIntegrable_cpow (#19877)

* `have : Ioc c 0 = Ioo c 0 ∪ {(0 : ℝ)} `  is directly proved by `(Ioo_union_right hc).symm`
* That shorter proof can then be inlined at its use in the `simp` in the next line.

This simplification was found by [`tryAtEachStep`](https://github.com/dwrensha/tryAtEachStep).
  • Loading branch information
dwrensha committed Dec 11, 2024
1 parent d840f50 commit 868f349
Showing 1 changed file with 1 addition and 4 deletions.
5 changes: 1 addition & 4 deletions Mathlib/Analysis/SpecialFunctions/Integrals.lean
Original file line number Diff line number Diff line change
Expand Up @@ -140,10 +140,7 @@ theorem intervalIntegrable_cpow {r : ℂ} (h : 0 ≤ r.re ∨ (0 : ℝ) ∉ [[a,
· -- case `c < 0`: integrand is identically constant, *except* at `x = 0` if `r ≠ 0`.
apply IntervalIntegrable.symm
rw [intervalIntegrable_iff_integrableOn_Ioc_of_le hc.le]
have : Ioc c 0 = Ioo c 0 ∪ {(0 : ℝ)} := by
rw [← Ioo_union_Icc_eq_Ioc hc (le_refl 0), ← Icc_def]
simp_rw [← le_antisymm_iff, setOf_eq_eq_singleton']
rw [this, integrableOn_union, and_comm]; constructor
rw [← Ioo_union_right hc, integrableOn_union, and_comm]; constructor
· refine integrableOn_singleton_iff.mpr (Or.inr ?_)
exact isFiniteMeasureOnCompacts_of_isLocallyFiniteMeasure.lt_top_of_isCompact
isCompact_singleton
Expand Down

0 comments on commit 868f349

Please sign in to comment.