Skip to content

Commit

Permalink
chore: no need to pass autoParam to simp or dsimp (#15968)
Browse files Browse the repository at this point in the history
and with leanprover/lean4#4154 it actually
complains, so let's remove them now.
  • Loading branch information
nomeata authored and bjoernkjoshanssen committed Sep 9, 2024
1 parent 868f961 commit f4cd7f2
Show file tree
Hide file tree
Showing 5 changed files with 13 additions and 13 deletions.
12 changes: 6 additions & 6 deletions Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -256,29 +256,29 @@ open Opposite
-- Porting note: simp wasn't firing but rw was, annoying
instance : MonoidalPreadditive (ModuleCat.{u} R) := by
refine ⟨?_, ?_, ?_, ?_⟩
· dsimp only [autoParam]; intros
· intros
refine TensorProduct.ext (LinearMap.ext fun x => LinearMap.ext fun y => ?_)
simp only [LinearMap.compr₂_apply, TensorProduct.mk_apply]
rw [LinearMap.zero_apply]
-- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
erw [MonoidalCategory.whiskerLeft_apply]
rw [LinearMap.zero_apply, TensorProduct.tmul_zero]
· dsimp only [autoParam]; intros
· intros
refine TensorProduct.ext (LinearMap.ext fun x => LinearMap.ext fun y => ?_)
simp only [LinearMap.compr₂_apply, TensorProduct.mk_apply]
rw [LinearMap.zero_apply]
-- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
erw [MonoidalCategory.whiskerRight_apply]
rw [LinearMap.zero_apply, TensorProduct.zero_tmul]
· dsimp only [autoParam]; intros
· intros
refine TensorProduct.ext (LinearMap.ext fun x => LinearMap.ext fun y => ?_)
simp only [LinearMap.compr₂_apply, TensorProduct.mk_apply]
rw [LinearMap.add_apply]
-- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
erw [MonoidalCategory.whiskerLeft_apply, MonoidalCategory.whiskerLeft_apply]
erw [MonoidalCategory.whiskerLeft_apply]
rw [LinearMap.add_apply, TensorProduct.tmul_add]
· dsimp only [autoParam]; intros
· intros
refine TensorProduct.ext (LinearMap.ext fun x => LinearMap.ext fun y => ?_)
simp only [LinearMap.compr₂_apply, TensorProduct.mk_apply]
rw [LinearMap.add_apply]
Expand All @@ -290,14 +290,14 @@ instance : MonoidalPreadditive (ModuleCat.{u} R) := by
-- Porting note: simp wasn't firing but rw was, annoying
instance : MonoidalLinear R (ModuleCat.{u} R) := by
refine ⟨?_, ?_⟩
· dsimp only [autoParam]; intros
· intros
refine TensorProduct.ext (LinearMap.ext fun x => LinearMap.ext fun y => ?_)
simp only [LinearMap.compr₂_apply, TensorProduct.mk_apply]
rw [LinearMap.smul_apply]
-- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
erw [MonoidalCategory.whiskerLeft_apply, MonoidalCategory.whiskerLeft_apply]
rw [LinearMap.smul_apply, TensorProduct.tmul_smul]
· dsimp only [autoParam]; intros
· intros
refine TensorProduct.ext (LinearMap.ext fun x => LinearMap.ext fun y => ?_)
simp only [LinearMap.compr₂_apply, TensorProduct.mk_apply]
rw [LinearMap.smul_apply]
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/DifferentialObject.lean
Original file line number Diff line number Diff line change
Expand Up @@ -181,8 +181,8 @@ def mapDifferentialObject (F : C ⥤ D)
slice_lhs 2 3 => rw [← Functor.comp_map F (shiftFunctor D (1 : S)), ← η.naturality f.f]
slice_lhs 1 2 => rw [Functor.comp_map, ← F.map_comp, f.comm, F.map_comp]
rw [Category.assoc] }
map_id := by intros; ext; simp [autoParam]
map_comp := by intros; ext; simp [autoParam]
map_id := by intros; ext; simp
map_comp := by intros; ext; simp

end Functor

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Elements.lean
Original file line number Diff line number Diff line change
Expand Up @@ -265,7 +265,7 @@ theorem costructuredArrow_yoneda_equivalence_naturality {F₁ F₂ : Cᵒᵖ ⥤
congr
ext _ f
simpa using congr_fun (α.naturality f.op).symm (unop X).snd
· simp [autoParam]
· simp

/-- The equivalence `F.elementsᵒᵖ ≌ (yoneda, F)` is compatible with the forgetful functors. -/
@[simps!]
Expand Down
6 changes: 3 additions & 3 deletions Mathlib/Data/List/Intervals.lean
Original file line number Diff line number Diff line change
Expand Up @@ -42,15 +42,15 @@ theorem zero_bot (n : ℕ) : Ico 0 n = range n := by rw [Ico, Nat.sub_zero, rang
@[simp]
theorem length (n m : ℕ) : length (Ico n m) = m - n := by
dsimp [Ico]
simp [length_range', autoParam]
simp [length_range']

theorem pairwise_lt (n m : ℕ) : Pairwise (· < ·) (Ico n m) := by
dsimp [Ico]
simp [pairwise_lt_range', autoParam]
simp [pairwise_lt_range']

theorem nodup (n m : ℕ) : Nodup (Ico n m) := by
dsimp [Ico]
simp [nodup_range', autoParam]
simp [nodup_range']

@[simp]
theorem mem {n m l : ℕ} : l ∈ Ico n m ↔ n ≤ l ∧ l < m := by
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Sheaves/Presheaf.lean
Original file line number Diff line number Diff line change
Expand Up @@ -303,7 +303,7 @@ def pullbackObjObjOfImageOpen {X Y : TopCat.{v}} (f : X ⟶ Y) (ℱ : Y.Presheaf
refine (homOfLE ?_).op
apply (Set.image_subset f s.pt.hom.unop.le).trans
exact Set.image_preimage.l_u_le (SetLike.coe s.pt.left.unop)
· simp [autoParam, eq_iff_true_of_subsingleton] }
· simp [eq_iff_true_of_subsingleton] }
exact IsColimit.coconePointUniqueUpToIso
((Opens.map f).op.isPointwiseLeftKanExtensionLanUnit ℱ (op U))
(colimitOfDiagramTerminal hx _)
Expand Down

0 comments on commit f4cd7f2

Please sign in to comment.