Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
FLDutchmann committed Feb 11, 2025
1 parent 2a2caee commit ca24083
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/Mertens.lean
Original file line number Diff line number Diff line change
Expand Up @@ -611,7 +611,7 @@ theorem integrableOn_Ici_fun_mul_E₁ (t : ℝ) (ht : 1 < t) :
measurableSet_Ici
have := isBigO.integrableAtFilter («μ» := volume) (mul_E₁_measurable.stronglyMeasurable.stronglyMeasurableAtFilter)
(integrable_inv_mul_log_inv_sq t ht).integrableAtFilter
rw [integrableAtFilter_principal_iff] at this
rw [_root_.integrableAtFilter_principal_iff] at this
exact this

theorem integral_mul_E₁_eq_const_sub_integral (x a : ℝ) (ha : 1 < a) (hx : a ≤ x) :
Expand Down

0 comments on commit ca24083

Please sign in to comment.