Skip to content

Commit

Permalink
more timeouts
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Apr 4, 2024
1 parent f2540a1 commit 269f6b2
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Mathlib/Analysis/Fourier/FourierTransformDeriv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -107,6 +107,9 @@ lemma norm_fourierSMulRight_le (L : V →L[ℝ] W →L[ℝ] ℝ) (f : V → E) (
_ ≤ (2 * π) * (‖L‖ * ‖v‖) * ‖f v‖ := by gcongr; exact L.le_opNorm _
_ = 2 * π * ‖L‖ * ‖v‖ * ‖f v‖ := by ring

-- Adaptation note: nightly-2024-04-01
-- This maxHeartbeats was not needed previously.
set_option maxHeartbeats 400000 in
lemma _root_.MeasureTheory.AEStronglyMeasurable.fourierSMulRight
[SecondCountableTopologyEither V (W →L[ℝ] ℝ)] [MeasurableSpace V] [BorelSpace V]
{L : V →L[ℝ] W →L[ℝ] ℝ} {f : V → E} {μ : Measure V}
Expand Down
3 changes: 3 additions & 0 deletions Mathlib/Probability/Kernel/MeasureCompProd.lean
Original file line number Diff line number Diff line change
Expand Up @@ -69,6 +69,9 @@ lemma ae_compProd_of_ae_ae [SFinite μ] [IsSFiniteKernel κ] {p : α × β → P
∀ᵐ x ∂(μ ⊗ₘ κ), p x :=
kernel.ae_compProd_of_ae_ae hp h

-- Adaptation note: nightly-2024-04-01
-- This maxHeartbeats was not needed previously.
set_option maxHeartbeats 400000 in
lemma ae_ae_of_ae_compProd [SFinite μ] [IsSFiniteKernel κ] {p : α × β → Prop}
(h : ∀ᵐ x ∂(μ ⊗ₘ κ), p x) :
∀ᵐ a ∂μ, ∀ᵐ b ∂(κ a), p (a, b) :=
Expand Down

0 comments on commit 269f6b2

Please sign in to comment.