Skip to content

Commit

Permalink
chore: classify used to be dsimp porting notes (#10935)
Browse files Browse the repository at this point in the history
Classifies by adding issue number (#10934) to porting notes claiming anything semantically equivalent to: 

- "used to be `dsimp`"
- "was `dsimp`"
  • Loading branch information
pitmonticone committed Feb 27, 2024
1 parent d8fa853 commit 87798ab
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 8 deletions.
10 changes: 5 additions & 5 deletions Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean
Expand Up @@ -99,7 +99,7 @@ theorem μ_natural {X Y X' Y' : Type u} (f : X ⟶ Y) (g : X' ⟶ Y') :
apply LinearMap.ext_ring
apply Finsupp.ext
intro ⟨y, y'⟩
-- Porting note: used to be dsimp [μ]
-- Porting note (#10934): used to be dsimp [μ]
change (finsuppTensorFinsupp' R Y Y')
(Finsupp.mapDomain f (Finsupp.single x 1) ⊗ₜ[R] Finsupp.mapDomain g (Finsupp.single x' 1)) _
= (Finsupp.mapDomain (f ⊗ g) (finsuppTensorFinsupp' R X X'
Expand All @@ -122,7 +122,7 @@ theorem left_unitality (X : Type u) :
apply LinearMap.ext_ring
apply Finsupp.ext
intro x'
-- Porting note: used to be dsimp [ε, μ]
-- Porting note (#10934): used to be dsimp [ε, μ]
let q : X →₀ R := ((λ_ (of R (X →₀ R))).hom) (1 ⊗ₜ[R] Finsupp.single x 1)
change q x' = Finsupp.mapDomain (λ_ X).hom (finsuppTensorFinsupp' R (𝟙_ (Type u)) X
(Finsupp.single PUnit.unit 1 ⊗ₜ[R] Finsupp.single x 1)) x'
Expand All @@ -143,7 +143,7 @@ theorem right_unitality (X : Type u) :
apply LinearMap.ext_ring
apply Finsupp.ext
intro x'
-- Porting note: used to be dsimp [ε, μ]
-- Porting note (#10934): used to be dsimp [ε, μ]
let q : X →₀ R := ((ρ_ (of R (X →₀ R))).hom) (Finsupp.single x 1 ⊗ₜ[R] 1)
change q x' = Finsupp.mapDomain (ρ_ X).hom (finsuppTensorFinsupp' R X (𝟙_ (Type u))
(Finsupp.single x 1 ⊗ₜ[R] Finsupp.single PUnit.unit 1)) x'
Expand Down Expand Up @@ -171,7 +171,7 @@ theorem associativity (X Y Z : Type u) :
apply LinearMap.ext_ring
apply Finsupp.ext
intro a
-- Porting note: used to be dsimp [μ]
-- Porting note (#10934): used to be dsimp [μ]
change Finsupp.mapDomain (α_ X Y Z).hom (finsuppTensorFinsupp' R (X ⊗ Y) Z
(finsuppTensorFinsupp' R X Y
(Finsupp.single x 1 ⊗ₜ[R] Finsupp.single y 1) ⊗ₜ[R] Finsupp.single z 1)) a =
Expand Down Expand Up @@ -224,7 +224,7 @@ variable [CommRing R]
/-- The free functor `Type u ⥤ ModuleCat R`, as a monoidal functor. -/
def monoidalFree : MonoidalFunctor (Type u) (ModuleCat.{u} R) :=
{ LaxMonoidalFunctor.of (free R).obj with
-- Porting note: used to be dsimp
-- Porting note (#10934): used to be dsimp
ε_isIso := (by infer_instance : IsIso (@LaxMonoidal.ε _ _ _ _ _ _ (free R).obj _ _))
μ_isIso := fun X Y => by dsimp; infer_instance }
#align Module.monoidal_free ModuleCat.monoidalFree
Expand Down
6 changes: 3 additions & 3 deletions Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean
Expand Up @@ -168,7 +168,7 @@ theorem leftUnitor_naturality {M N : ModuleCat R} (f : M ⟶ N) :
apply TensorProduct.ext
apply LinearMap.ext_ring
apply LinearMap.ext; intro x
-- Porting note: used to be dsimp
-- Porting note (#10934): used to be dsimp
change ((leftUnitor N).hom) ((tensorHom (𝟙 (of R R)) f) ((1 : R) ⊗ₜ[R] x)) =
f (((leftUnitor M).hom) (1 ⊗ₜ[R] x))
erw [TensorProduct.lid_tmul, TensorProduct.lid_tmul]
Expand All @@ -182,7 +182,7 @@ theorem rightUnitor_naturality {M N : ModuleCat R} (f : M ⟶ N) :
apply TensorProduct.ext
apply LinearMap.ext; intro x
apply LinearMap.ext_ring
-- Porting note: used to be dsimp
-- Porting note (#10934): used to be dsimp
change ((rightUnitor N).hom) ((tensorHom f (𝟙 (of R R))) (x ⊗ₜ[R] (1 : R))) =
f (((rightUnitor M).hom) (x ⊗ₜ[R] 1))
erw [TensorProduct.rid_tmul, TensorProduct.rid_tmul]
Expand All @@ -196,7 +196,7 @@ theorem triangle (M N : ModuleCat.{u} R) :
apply TensorProduct.ext_threefold
intro x y z
change R at y
-- Porting note: used to be dsimp [tensorHom, associator]
-- Porting note (#10934): used to be dsimp [tensorHom, associator]
change x ⊗ₜ[R] ((leftUnitor N).hom) (y ⊗ₜ[R] z) = ((rightUnitor M).hom) (x ⊗ₜ[R] y) ⊗ₜ[R] z
erw [TensorProduct.lid_tmul, TensorProduct.rid_tmul]
exact (TensorProduct.smul_tmul _ _ _).symm
Expand Down

0 comments on commit 87798ab

Please sign in to comment.