Skip to content

Commit

Permalink
zetaDelta
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 21, 2024
1 parent b1016a1 commit 8964f49
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Sites/Over.lean
Original file line number Diff line number Diff line change
Expand Up @@ -77,7 +77,7 @@ lemma overEquiv_pullback {X : C} {Y₁ Y₂ : Over X} (f : Y₁ ⟶ Y₂) (S : S
let T := Over.mk (b ≫ W.hom)
let c : T ⟶ Y₁ := Over.homMk g (by dsimp [T]; rw [← Over.w a, ← reassoc_of% w, Over.w f])
let d : T ⟶ W := Over.homMk b
refine ⟨T, c, 𝟙 Z, ?_, by simp [c]⟩
refine ⟨T, c, 𝟙 Z, ?_, by simp +zetaDelta [c]⟩
rw [show c ≫ f = d ≫ a by ext; exact w]
exact S.downward_closed h _

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/MeasurableSpace/Embedding.lean
Original file line number Diff line number Diff line change
Expand Up @@ -722,7 +722,7 @@ noncomputable def schroederBernstein {f : α → β} {g : β → α} (hf : Measu
have : Aᶜ = g '' Bᶜ := by
apply compl_injective
rw [← Afp]
simp
simp +zetaDelta
rw [this]
exact (hg.equivImage _).symm
have Fmono : ∀ {A B}, A ⊆ B → F A ⊆ F B := fun h =>
Expand Down

0 comments on commit 8964f49

Please sign in to comment.