Skip to content

Commit

Permalink
fix: don't zeta-expand in filter_upwards (#7213)
Browse files Browse the repository at this point in the history
  • Loading branch information
PatrickMassot committed Sep 17, 2023
1 parent 8b0612f commit 1937612
Show file tree
Hide file tree
Showing 5 changed files with 4 additions and 2 deletions.
1 change: 1 addition & 0 deletions Mathlib/MeasureTheory/Integral/FundThmCalculus.lean
Expand Up @@ -1217,6 +1217,7 @@ theorem integral_eq_sub_of_hasDerivAt_of_tendsto (hab : a < b) {fa fb}
have Fderiv : ∀ x ∈ Ioo a b, HasDerivAt F (f' x) x := by
refine' fun x hx => (hderiv x hx).congr_of_eventuallyEq _
filter_upwards [Ioo_mem_nhds hx.1 hx.2] with _ hy
unfold_let F
rw [update_noteq hy.2.ne, update_noteq hy.1.ne']
have hcont : ContinuousOn F (Icc a b) := by
rw [continuousOn_update_iff, continuousOn_update_iff, Icc_diff_right, Ico_diff_left]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/Filter/Basic.lean
Expand Up @@ -266,7 +266,7 @@ elab_rules : tactic
return [m.mvarId!]
liftMetaTactic fun goal => do
goal.apply (← mkConstWithFreshMVarLevels ``Filter.univ_mem') config
evalTactic <|← `(tactic| dsimp only [Set.mem_setOf_eq])
evalTactic <|← `(tactic| dsimp (config := {zeta := false}) only [Set.mem_setOf_eq])
if let some l := wth then
evalTactic <|← `(tactic| intro $[$l]*)
if let some e := usingArg then
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Probability/Independence/Kernel.lean
Expand Up @@ -553,7 +553,6 @@ theorem iIndepSets.piiUnionInter_of_not_mem {π : ι → Set (Set Ω)} {a : ι}
have has : a ∉ s := fun has_mem => haS (hs_mem has_mem)
filter_upwards [h_μ_t1, h_μ_inter] with a' ha1 ha2
rw [ha2, Finset.prod_insert has, h_t2, mul_comm, ha1]
simp only [ite_true]

/-- The measurable space structures generated by independent pi-systems are independent. -/
theorem iIndepSets.iIndep [IsMarkovKernel κ] (m : ι → MeasurableSpace Ω)
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Probability/Martingale/Centering.lean
Expand Up @@ -147,6 +147,7 @@ theorem martingalePart_add_ae_eq [SigmaFiniteFiltration μ ℱ] {f g : ℕ →
(hf.integrable n).add <| hgint n)
refine' (eventuallyEq_iff_sub.2 _).symm
filter_upwards [hhmgle.eq_zero_of_predictable hhpred n] with ω hω
unfold_let h at hω
rw [Pi.sub_apply] at hω
rw [hω, Pi.sub_apply, martingalePart]
simp [hg0]
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Topology/DenseEmbedding.lean
Expand Up @@ -201,6 +201,7 @@ theorem continuousAt_extend [T3Space γ] {b : β} {f : α → γ} (di : DenseInd
have V₁_in : V₁ ∈ 𝓝 b := by
filter_upwards [hf]
rintro x ⟨c, hc⟩
unfold_let φ
rwa [di.extend_eq_of_tendsto hc]
obtain ⟨V₂, V₂_in, V₂_op, hV₂⟩ : ∃ V₂ ∈ 𝓝 b, IsOpen V₂ ∧ ∀ x ∈ i ⁻¹' V₂, f x ∈ V' := by
simpa [and_assoc] using
Expand Down

0 comments on commit 1937612

Please sign in to comment.