Skip to content

Commit

Permalink
chore: remove redundant dsimp args (#9835)
Browse files Browse the repository at this point in the history
This is needed to work with leanprover/lean4#3087
  • Loading branch information
marcusrossel committed Jan 18, 2024
1 parent 05dc888 commit a5e04cb
Show file tree
Hide file tree
Showing 7 changed files with 7 additions and 7 deletions.
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Limits/Presheaf.lean
Expand Up @@ -390,7 +390,7 @@ noncomputable def natIsoOfNatIsoOnRepresentables (L₁ L₂ : (Cᵒᵖ ⥤ Type
· intro P₁ P₂ f
apply (isColimitOfPreserves L₁ (colimitOfRepresentable P₁)).hom_ext
intro j
dsimp only [id.def, IsColimit.comp_coconePointsIsoOfNatIso_hom, isoWhiskerLeft_hom]
dsimp only [id.def, isoWhiskerLeft_hom]
have :
(L₁.mapCocone (coconeOfRepresentable P₁)).ι.app j ≫ L₁.map f =
(L₁.mapCocone (coconeOfRepresentable P₂)).ι.app
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Limits/Shapes/Pullbacks.lean
Expand Up @@ -616,7 +616,7 @@ theorem equalizer_ext (t : PullbackCone f g) {W : C} {k l : W ⟶ t.pt} (h₀ :
(h₁ : k ≫ snd t = l ≫ snd t) : ∀ j : WalkingCospan, k ≫ t.π.app j = l ≫ t.π.app j
| some WalkingPair.left => h₀
| some WalkingPair.right => h₁
| none => by rw [← t.w inl]; dsimp [h₀]; simp only [← Category.assoc, congrArg (· ≫ f) h₀]
| none => by rw [← t.w inl, reassoc_of% h₀]
#align category_theory.limits.pullback_cone.equalizer_ext CategoryTheory.Limits.PullbackCone.equalizer_ext

theorem IsLimit.hom_ext {t : PullbackCone f g} (ht : IsLimit t) {W : C} {k l : W ⟶ t.pt}
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Complex/Exponential.lean
Expand Up @@ -549,7 +549,7 @@ theorem exp_conj : exp (conj x) = conj (exp x) := by
dsimp [exp]
rw [← lim_conj]
refine' congr_arg CauSeq.lim (CauSeq.ext fun _ => _)
dsimp [exp', Function.comp_def, isCauSeq_conj, cauSeqConj]
dsimp [exp', Function.comp_def, cauSeqConj]
rw [(starRingEnd _).map_sum]
refine' sum_congr rfl fun n _ => _
rw [map_div₀, map_pow, ← ofReal_nat_cast, conj_ofReal]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/List/Perm.lean
Expand Up @@ -746,7 +746,7 @@ theorem perm_permutations'Aux_comm (a b : α) (l : List α) :
theorem Perm.permutations' {s t : List α} (p : s ~ t) : permutations' s ~ permutations' t := by
induction' p with a s t _ IH a b l s t u _ _ IH₁ IH₂; · simp
· exact IH.bind_right _
· dsimp [permutations']
· dsimp
rw [bind_assoc, bind_assoc]
apply Perm.bind_left
intro l' _
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/ZMod/Basic.lean
Expand Up @@ -819,7 +819,7 @@ def chineseRemainder {m n : ℕ} (h : m.Coprime n) : ZMod (m * n) ≃+* ZMod m
haveI : NeZero n := ⟨right_ne_zero_of_mul hmn0⟩
have left_inv : Function.LeftInverse inv_fun to_fun := by
intro x
dsimp only [dvd_mul_left, dvd_mul_right, ZMod.castHom_apply]
dsimp only [ZMod.castHom_apply]
conv_rhs => rw [← ZMod.nat_cast_zmod_val x]
rw [if_neg hmn0, ZMod.eq_iff_modEq_nat, ← Nat.modEq_and_modEq_iff_modEq_mul h,
Prod.fst_zmod_cast, Prod.snd_zmod_cast]
Expand Down
Expand Up @@ -627,7 +627,7 @@ theorem forget₂ToModuleCatHomotopyEquiv_f_0_eq :
simp only [HomologicalComplex.comp_f]
dsimp
convert Category.id_comp (X := (forget₂ToModuleCat k G).X 0) _
· dsimp only [HomotopyEquiv.ofIso, compForgetAugmentedIso, map_alternatingFaceMapComplex]
· dsimp only [HomotopyEquiv.ofIso, compForgetAugmentedIso]
simp only [Iso.symm_hom, eqToIso.inv, HomologicalComplex.eqToHom_f, eqToHom_refl]
trans (Finsupp.total _ _ _ fun _ => (1 : k)).comp ((ModuleCat.free k).map (terminal.from _))
· dsimp
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/SetTheory/Game/PGame.lean
Expand Up @@ -1663,7 +1663,7 @@ theorem neg_add_le {x y : PGame} : -(x + y) ≤ -x + -y :=
def addCommRelabelling : ∀ x y : PGame.{u}, x + y ≡r y + x
| mk xl xr xL xR, mk yl yr yL yR => by
refine' ⟨Equiv.sumComm _ _, Equiv.sumComm _ _, _, _⟩ <;> rintro (_ | _) <;>
· dsimp [leftMoves_add, rightMoves_add]
· dsimp
apply addCommRelabelling
termination_by _ x y => (x, y)
#align pgame.add_comm_relabelling SetTheory.PGame.addCommRelabelling
Expand Down

0 comments on commit a5e04cb

Please sign in to comment.