Skip to content

Commit

Permalink
fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jan 5, 2025
1 parent a340252 commit 0c2797e
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Abelian/InjectiveResolution.lean
Original file line number Diff line number Diff line change
Expand Up @@ -240,7 +240,7 @@ lemma InjectiveResolution.iso_hom_naturality {X Y : C} (f : X ⟶ Y)
I.iso.hom ≫ (HomotopyCategory.quotient _ _).map φ := by
apply HomotopyCategory.eq_of_homotopy
apply descHomotopy f
simp
all_goals aesop

@[reassoc]
lemma InjectiveResolution.iso_inv_naturality {X Y : C} (f : X ⟶ Y)
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Limits/Shapes/Pullback/Square.lean
Original file line number Diff line number Diff line change
Expand Up @@ -79,7 +79,7 @@ lemma IsPullback.of_iso {sq₁ sq₂ : Square C} (h : sq₁.IsPullback)
refine CategoryTheory.IsPullback.of_iso h
(evaluation₁.mapIso e) (evaluation₂.mapIso e)
(evaluation₃.mapIso e) (evaluation₄.mapIso e) ?_ ?_ ?_ ?_
simp
all_goals simp

lemma IsPullback.iff_of_iso {sq₁ sq₂ : Square C} (e : sq₁ ≅ sq₂) :
sq₁.IsPullback ↔ sq₂.IsPullback :=
Expand All @@ -90,7 +90,7 @@ lemma IsPushout.of_iso {sq₁ sq₂ : Square C} (h : sq₁.IsPushout)
refine CategoryTheory.IsPushout.of_iso h
(evaluation₁.mapIso e) (evaluation₂.mapIso e)
(evaluation₃.mapIso e) (evaluation₄.mapIso e) ?_ ?_ ?_ ?_
simp
all_goals simp

lemma IsPushout.iff_of_iso {sq₁ sq₂ : Square C} (e : sq₁ ≅ sq₂) :
sq₁.IsPushout ↔ sq₂.IsPushout :=
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Probability/StrongLaw.lean
Original file line number Diff line number Diff line change
Expand Up @@ -426,7 +426,7 @@ theorem strong_law_aux1 {c : ℝ} (c_one : 1 < c) {ε : ℝ} (εpos : 0 < ε) :
· simp only [mem_sigma, mem_range, filter_congr_decidable, mem_filter, and_imp,
Sigma.forall]
exact fun a b haN hb ↦ ⟨hb.trans_le <| u_mono <| Nat.le_pred_of_lt haN, haN, hb⟩
simp
all_goals simp
_ ≤ ∑ j ∈ range (u (N - 1)), c ^ 5 * (c - 1)⁻¹ ^ 3 / ↑j ^ 2 * Var[Y j] := by
apply sum_le_sum fun j hj => ?_
rcases @eq_zero_or_pos _ _ j with (rfl | hj)
Expand Down

0 comments on commit 0c2797e

Please sign in to comment.