algebra.category.Module.monoidal.closed
⟷
Mathlib.Algebra.Category.ModuleCat.Monoidal.Closed
The following section lists changes to this file in mathlib3 and mathlib4 that occured after the initial port. Most recent changes are shown first. Hovering over a commit will show all commits associated with the same mathlib3 commit.
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(last sync)
mathlib commit https://github.com/leanprover-community/mathlib/commit/65a1391a0106c9204fe45bc73a039f056558cb83
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Scott Morrison, Jakob von Raumer
-/
import CategoryTheory.Closed.Monoidal
-import Algebra.Category.Module.Monoidal.Symmetric
+import Algebra.Category.ModuleCat.Monoidal.Symmetric
#align_import algebra.category.Module.monoidal.closed from "leanprover-community/mathlib"@"c20927220ef87bb4962ba08bf6da2ce3cf50a6dd"
mathlib commit https://github.com/leanprover-community/mathlib/commit/ce64cd319bb6b3e82f31c2d38e79080d377be451
@@ -3,8 +3,8 @@ Copyright (c) 2020 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Scott Morrison, Jakob von Raumer
-/
-import Mathbin.CategoryTheory.Closed.Monoidal
-import Mathbin.Algebra.Category.Module.Monoidal.Symmetric
+import CategoryTheory.Closed.Monoidal
+import Algebra.Category.Module.Monoidal.Symmetric
#align_import algebra.category.Module.monoidal.closed from "leanprover-community/mathlib"@"c20927220ef87bb4962ba08bf6da2ce3cf50a6dd"
mathlib commit https://github.com/leanprover-community/mathlib/commit/8ea5598db6caeddde6cb734aa179cc2408dbd345
@@ -2,15 +2,12 @@
Copyright (c) 2020 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Scott Morrison, Jakob von Raumer
-
-! This file was ported from Lean 3 source module algebra.category.Module.monoidal.closed
-! leanprover-community/mathlib commit c20927220ef87bb4962ba08bf6da2ce3cf50a6dd
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
-/
import Mathbin.CategoryTheory.Closed.Monoidal
import Mathbin.Algebra.Category.Module.Monoidal.Symmetric
+#align_import algebra.category.Module.monoidal.closed from "leanprover-community/mathlib"@"c20927220ef87bb4962ba08bf6da2ce3cf50a6dd"
+
/-!
# The monoidal closed structure on `Module R`.
mathlib commit https://github.com/leanprover-community/mathlib/commit/2a0ce625dbb0ffbc7d1316597de0b25c1ec75303
@@ -43,11 +43,11 @@ def monoidalClosedHomEquiv (M N P : ModuleCat.{u} R) :
toFun f := LinearMap.compr₂ (TensorProduct.mk R N M) ((β_ N M).Hom ≫ f)
invFun f := (β_ M N).Hom ≫ TensorProduct.lift f
left_inv f := by
- ext (m n)
+ ext m n
simp only [TensorProduct.mk_apply, TensorProduct.lift.tmul, LinearMap.compr₂_apply,
Function.comp_apply, coe_comp, monoidal_category.braiding_hom_apply]
right_inv f := by
- ext (m n)
+ ext m n
simp only [TensorProduct.mk_apply, TensorProduct.lift.tmul, LinearMap.compr₂_apply,
symmetric_category.symmetry_assoc]
#align Module.monoidal_closed_hom_equiv ModuleCat.monoidalClosedHomEquiv
mathlib commit https://github.com/leanprover-community/mathlib/commit/9fb8964792b4237dac6200193a0d533f1b3f7423
@@ -31,6 +31,7 @@ variable {R : Type u} [CommRing R]
attribute [local ext] TensorProduct.ext
+#print ModuleCat.monoidalClosedHomEquiv /-
/-- Auxiliary definition for the `monoidal_closed` instance on `Module R`.
(This is only a separate definition in order to speed up typechecking. )
-/
@@ -50,6 +51,7 @@ def monoidalClosedHomEquiv (M N P : ModuleCat.{u} R) :
simp only [TensorProduct.mk_apply, TensorProduct.lift.tmul, LinearMap.compr₂_apply,
symmetric_category.symmetry_assoc]
#align Module.monoidal_closed_hom_equiv ModuleCat.monoidalClosedHomEquiv
+-/
instance : MonoidalClosed (ModuleCat.{u} R)
where closed' M :=
@@ -58,12 +60,15 @@ instance : MonoidalClosed (ModuleCat.{u} R)
{ right := (linearCoyoneda R (ModuleCat.{u} R)).obj (op M)
adj := Adjunction.mkOfHomEquiv { homEquiv := fun N P => monoidalClosedHomEquiv M N P } } }
+#print ModuleCat.ihom_map_apply /-
theorem ihom_map_apply {M N P : ModuleCat.{u} R} (f : N ⟶ P) (g : ModuleCat.of R (M ⟶ N)) :
(ihom M).map f g = g ≫ f :=
rfl
#align Module.ihom_map_apply ModuleCat.ihom_map_apply
+-/
/- ./././Mathport/Syntax/Translate/Expr.lean:177:8: unsupported: ambiguous notation -/
+#print ModuleCat.monoidalClosed_curry /-
-- I can't seem to express the function coercion here without writing `@coe_fn`.
@[simp]
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
@@ -71,13 +76,17 @@ theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x :
f (x ⊗ₜ[R] y) :=
rfl
#align Module.monoidal_closed_curry ModuleCat.monoidalClosed_curry
+-/
+#print ModuleCat.monoidalClosed_uncurry /-
@[simp]
theorem monoidalClosed_uncurry {M N P : ModuleCat.{u} R} (f : N ⟶ M ⟶[ModuleCat.{u} R] P) (x : M)
(y : N) : MonoidalClosed.uncurry f (x ⊗ₜ[R] y) = (@coeFn _ _ LinearMap.hasCoeToFun (f y)) x :=
rfl
#align Module.monoidal_closed_uncurry ModuleCat.monoidalClosed_uncurry
+-/
+#print ModuleCat.ihom_ev_app /-
/-- Describes the counit of the adjunction `M ⊗ - ⊣ Hom(M, -)`. Given an `R`-module `N` this
should give a map `M ⊗ Hom(M, N) ⟶ N`, so we flip the order of the arguments in the identity map
`Hom(M, N) ⟶ (M ⟶ N)` and uncurry the resulting map `M ⟶ Hom(M, N) ⟶ N.` -/
@@ -87,7 +96,9 @@ theorem ihom_ev_app (M N : ModuleCat.{u} R) :
ext
exact ModuleCat.monoidalClosed_uncurry _ _ _
#align Module.ihom_ev_app ModuleCat.ihom_ev_app
+-/
+#print ModuleCat.ihom_coev_app /-
/-- Describes the unit of the adjunction `M ⊗ - ⊣ Hom(M, -)`. Given an `R`-module `N` this should
define a map `N ⟶ Hom(M, M ⊗ N)`, which is given by flipping the arguments in the natural
`R`-bilinear map `M ⟶ N ⟶ M ⊗ N`. -/
@@ -95,11 +106,14 @@ theorem ihom_coev_app (M N : ModuleCat.{u} R) :
(ihom.coev M).app N = (TensorProduct.mk _ _ _).flip :=
rfl
#align Module.ihom_coev_app ModuleCat.ihom_coev_app
+-/
+#print ModuleCat.monoidalClosed_pre_app /-
theorem monoidalClosed_pre_app {M N : ModuleCat.{u} R} (P : ModuleCat.{u} R) (f : N ⟶ M) :
(MonoidalClosed.pre f).app P = LinearMap.lcomp R _ f :=
rfl
#align Module.monoidal_closed_pre_app ModuleCat.monoidalClosed_pre_app
+-/
end ModuleCat
mathlib commit https://github.com/leanprover-community/mathlib/commit/31c24aa72e7b3e5ed97a8412470e904f82b81004
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Scott Morrison, Jakob von Raumer
! This file was ported from Lean 3 source module algebra.category.Module.monoidal.closed
-! leanprover-community/mathlib commit 74403a3b2551b0970855e14ef5e8fd0d6af1bfc2
+! leanprover-community/mathlib commit c20927220ef87bb4962ba08bf6da2ce3cf50a6dd
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
@@ -13,6 +13,9 @@ import Mathbin.Algebra.Category.Module.Monoidal.Symmetric
/-!
# The monoidal closed structure on `Module R`.
+
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
-/
mathlib commit https://github.com/leanprover-community/mathlib/commit/95a87616d63b3cb49d3fe678d416fbe9c4217bf4
Homogenises porting notes via capitalisation and addition of whitespace.
It makes the following changes:
@@ -23,7 +23,7 @@ namespace ModuleCat
variable {R : Type u} [CommRing R]
--- porting note: removed @[simps] as the simpNF linter complains
+-- Porting note: removed @[simps] as the simpNF linter complains
/-- Auxiliary definition for the `MonoidalClosed` instance on `Module R`.
(This is only a separate definition in order to speed up typechecking. )
-/
@@ -50,7 +50,7 @@ instance : MonoidalClosed (ModuleCat.{u} R) where
{ right := (linearCoyoneda R (ModuleCat.{u} R)).obj (op M)
adj := Adjunction.mkOfHomEquiv
{ homEquiv := fun N P => monoidalClosedHomEquiv M N P
- -- porting note: this proof was automatic in mathlib3
+ -- Porting note: this proof was automatic in mathlib3
homEquiv_naturality_left_symm := by
intros
apply TensorProduct.ext'
@@ -65,7 +65,7 @@ set_option linter.uppercaseLean3 false in
open MonoidalCategory
--- porting note: `CoeFun` was replaced by `DFunLike`
+-- Porting note: `CoeFun` was replaced by `DFunLike`
-- I can't seem to express the function coercion here without writing `@DFunLike.coe`.
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
@DFunLike.coe _ _ _ LinearMap.instFunLike
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Scott Morrison, Jakob von Raumer
-/
import Mathlib.CategoryTheory.Closed.Monoidal
+import Mathlib.CategoryTheory.Linear.Yoneda
import Mathlib.Algebra.Category.ModuleCat.Monoidal.Symmetric
#align_import algebra.category.Module.monoidal.closed from "leanprover-community/mathlib"@"74403a3b2551b0970855e14ef5e8fd0d6af1bfc2"
FunLike
(#9833)
This follows up from #9785, which renamed FunLike
to DFunLike
, by introducing a new abbreviation FunLike F α β := DFunLike F α (fun _ => β)
, to make the non-dependent use of FunLike
easier.
I searched for the pattern DFunLike.*fun
and DFunLike.*λ
in all files to replace expressions of the form DFunLike F α (fun _ => β)
with FunLike F α β
. I did this everywhere except for extends
clauses for two reasons: it would conflict with #8386, and more importantly extends
must directly refer to a structure with no unfolding of def
s or abbrev
s.
@@ -67,7 +67,7 @@ open MonoidalCategory
-- porting note: `CoeFun` was replaced by `DFunLike`
-- I can't seem to express the function coercion here without writing `@DFunLike.coe`.
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
- @DFunLike.coe _ _ _ LinearMap.instDFunLike
+ @DFunLike.coe _ _ _ LinearMap.instFunLike
((MonoidalClosed.curry f : N →ₗ[R] M →ₗ[R] P) y) x = f (x ⊗ₜ[R] y) :=
rfl
set_option linter.uppercaseLean3 false in
@@ -77,7 +77,7 @@ set_option linter.uppercaseLean3 false in
theorem monoidalClosed_uncurry
{M N P : ModuleCat.{u} R} (f : N ⟶ M ⟶[ModuleCat.{u} R] P) (x : M) (y : N) :
MonoidalClosed.uncurry f (x ⊗ₜ[R] y) =
- @DFunLike.coe _ _ _ LinearMap.instDFunLike (f y) x :=
+ @DFunLike.coe _ _ _ LinearMap.instFunLike (f y) x :=
rfl
set_option linter.uppercaseLean3 false in
#align Module.monoidal_closed_uncurry ModuleCat.monoidalClosed_uncurry
FunLike
to DFunLike
(#9785)
This prepares for the introduction of a non-dependent synonym of FunLike, which helps a lot with keeping #8386 readable.
This is entirely search-and-replace in 680197f combined with manual fixes in 4145626, e900597 and b8428f8. The commands that generated this change:
sed -i 's/\bFunLike\b/DFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\btoFunLike\b/toDFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/import Mathlib.Data.DFunLike/import Mathlib.Data.FunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\bHom_FunLike\b/Hom_DFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\binstFunLike\b/instDFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\bfunLike\b/instDFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\btoo many metavariables to apply `fun_like.has_coe_to_fun`/too many metavariables to apply `DFunLike.hasCoeToFun`/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
@@ -64,10 +64,10 @@ set_option linter.uppercaseLean3 false in
open MonoidalCategory
--- porting note: `CoeFun` was replaced by `FunLike`
--- I can't seem to express the function coercion here without writing `@FunLike.coe`.
+-- porting note: `CoeFun` was replaced by `DFunLike`
+-- I can't seem to express the function coercion here without writing `@DFunLike.coe`.
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
- @FunLike.coe _ _ _ LinearMap.instFunLike
+ @DFunLike.coe _ _ _ LinearMap.instDFunLike
((MonoidalClosed.curry f : N →ₗ[R] M →ₗ[R] P) y) x = f (x ⊗ₜ[R] y) :=
rfl
set_option linter.uppercaseLean3 false in
@@ -77,7 +77,7 @@ set_option linter.uppercaseLean3 false in
theorem monoidalClosed_uncurry
{M N P : ModuleCat.{u} R} (f : N ⟶ M ⟶[ModuleCat.{u} R] P) (x : M) (y : N) :
MonoidalClosed.uncurry f (x ⊗ₜ[R] y) =
- @FunLike.coe _ _ _ LinearMap.instFunLike (f y) x :=
+ @DFunLike.coe _ _ _ LinearMap.instDFunLike (f y) x :=
rfl
set_option linter.uppercaseLean3 false in
#align Module.monoidal_closed_uncurry ModuleCat.monoidalClosed_uncurry
@@ -66,8 +66,6 @@ open MonoidalCategory
-- porting note: `CoeFun` was replaced by `FunLike`
-- I can't seem to express the function coercion here without writing `@FunLike.coe`.
--- These lemmas have always been bad (#7657), but lean4#2644 made `simp` start noticing
-@[simp, nolint simpNF]
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
@FunLike.coe _ _ _ LinearMap.instFunLike
((MonoidalClosed.curry f : N →ₗ[R] M →ₗ[R] P) y) x = f (x ⊗ₜ[R] y) :=
@@ -34,9 +34,11 @@ def monoidalClosedHomEquiv (M N P : ModuleCat.{u} R) :
left_inv f := by
apply TensorProduct.ext'
intro m n
- rw [coe_comp, Function.comp_apply, MonoidalCategory.braiding_hom_apply,
- TensorProduct.lift.tmul, LinearMap.compr₂_apply,
- TensorProduct.mk_apply, coe_comp, Function.comp_apply, MonoidalCategory.braiding_hom_apply]
+ -- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
+ erw [coe_comp]
+ rw [Function.comp_apply]
+ -- This used to be `rw` and was longer (?), but we need `erw` after leanprover/lean4#2644
+ erw [MonoidalCategory.braiding_hom_apply, TensorProduct.lift.tmul]
right_inv f := rfl
set_option linter.uppercaseLean3 false in
#align Module.monoidal_closed_hom_equiv ModuleCat.monoidalClosedHomEquiv
@@ -64,7 +66,8 @@ open MonoidalCategory
-- porting note: `CoeFun` was replaced by `FunLike`
-- I can't seem to express the function coercion here without writing `@FunLike.coe`.
-@[simp]
+-- These lemmas have always been bad (#7657), but lean4#2644 made `simp` start noticing
+@[simp, nolint simpNF]
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
@FunLike.coe _ _ _ LinearMap.instFunLike
((MonoidalClosed.curry f : N →ₗ[R] M →ₗ[R] P) y) x = f (x ⊗ₜ[R] y) :=
@@ -34,11 +34,9 @@ def monoidalClosedHomEquiv (M N P : ModuleCat.{u} R) :
left_inv f := by
apply TensorProduct.ext'
intro m n
- -- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
- erw [coe_comp]
- rw [Function.comp_apply]
- -- This used to be `rw` and was longer (?), but we need `erw` after leanprover/lean4#2644
- erw [MonoidalCategory.braiding_hom_apply, TensorProduct.lift.tmul]
+ rw [coe_comp, Function.comp_apply, MonoidalCategory.braiding_hom_apply,
+ TensorProduct.lift.tmul, LinearMap.compr₂_apply,
+ TensorProduct.mk_apply, coe_comp, Function.comp_apply, MonoidalCategory.braiding_hom_apply]
right_inv f := rfl
set_option linter.uppercaseLean3 false in
#align Module.monoidal_closed_hom_equiv ModuleCat.monoidalClosedHomEquiv
@@ -66,8 +64,7 @@ open MonoidalCategory
-- porting note: `CoeFun` was replaced by `FunLike`
-- I can't seem to express the function coercion here without writing `@FunLike.coe`.
--- These lemmas have always been bad (#7657), but lean4#2644 made `simp` start noticing
-@[simp, nolint simpNF]
+@[simp]
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
@FunLike.coe _ _ _ LinearMap.instFunLike
((MonoidalClosed.curry f : N →ₗ[R] M →ₗ[R] P) y) x = f (x ⊗ₜ[R] y) :=
@@ -34,9 +34,11 @@ def monoidalClosedHomEquiv (M N P : ModuleCat.{u} R) :
left_inv f := by
apply TensorProduct.ext'
intro m n
- rw [coe_comp, Function.comp_apply, MonoidalCategory.braiding_hom_apply,
- TensorProduct.lift.tmul, LinearMap.compr₂_apply,
- TensorProduct.mk_apply, coe_comp, Function.comp_apply, MonoidalCategory.braiding_hom_apply]
+ -- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
+ erw [coe_comp]
+ rw [Function.comp_apply]
+ -- This used to be `rw` and was longer (?), but we need `erw` after leanprover/lean4#2644
+ erw [MonoidalCategory.braiding_hom_apply, TensorProduct.lift.tmul]
right_inv f := rfl
set_option linter.uppercaseLean3 false in
#align Module.monoidal_closed_hom_equiv ModuleCat.monoidalClosedHomEquiv
@@ -64,7 +66,8 @@ open MonoidalCategory
-- porting note: `CoeFun` was replaced by `FunLike`
-- I can't seem to express the function coercion here without writing `@FunLike.coe`.
-@[simp]
+-- These lemmas have always been bad (#7657), but lean4#2644 made `simp` start noticing
+@[simp, nolint simpNF]
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
@FunLike.coe _ _ _ LinearMap.instFunLike
((MonoidalClosed.curry f : N →ₗ[R] M →ₗ[R] P) y) x = f (x ⊗ₜ[R] y) :=
@@ -12,6 +12,7 @@ import Mathlib.Algebra.Category.ModuleCat.Monoidal.Symmetric
# The monoidal closed structure on `Module R`.
-/
+suppress_compilation
universe v w x u
Per https://github.com/leanprover/lean4/issues/2343, we are going to need to change the automatic generation of instance names, as they become too long.
This PR ensures that everywhere in Mathlib that refers to an instance by name, that name is given explicitly, rather than being automatically generated.
There are four exceptions, which are now commented, with links to https://github.com/leanprover/lean4/issues/2343.
This was implemented by running Mathlib against a modified Lean that appended _ᾰ
to all automatically generated names, and fixing everything.
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
@@ -65,7 +65,7 @@ open MonoidalCategory
-- I can't seem to express the function coercion here without writing `@FunLike.coe`.
@[simp]
theorem monoidalClosed_curry {M N P : ModuleCat.{u} R} (f : M ⊗ N ⟶ P) (x : M) (y : N) :
- @FunLike.coe _ _ _ LinearMap.instFunLikeLinearMap
+ @FunLike.coe _ _ _ LinearMap.instFunLike
((MonoidalClosed.curry f : N →ₗ[R] M →ₗ[R] P) y) x = f (x ⊗ₜ[R] y) :=
rfl
set_option linter.uppercaseLean3 false in
@@ -75,7 +75,7 @@ set_option linter.uppercaseLean3 false in
theorem monoidalClosed_uncurry
{M N P : ModuleCat.{u} R} (f : N ⟶ M ⟶[ModuleCat.{u} R] P) (x : M) (y : N) :
MonoidalClosed.uncurry f (x ⊗ₜ[R] y) =
- @FunLike.coe _ _ _ LinearMap.instFunLikeLinearMap (f y) x :=
+ @FunLike.coe _ _ _ LinearMap.instFunLike (f y) x :=
rfl
set_option linter.uppercaseLean3 false in
#align Module.monoidal_closed_uncurry ModuleCat.monoidalClosed_uncurry
@@ -2,15 +2,12 @@
Copyright (c) 2020 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Scott Morrison, Jakob von Raumer
-
-! This file was ported from Lean 3 source module algebra.category.Module.monoidal.closed
-! leanprover-community/mathlib commit 74403a3b2551b0970855e14ef5e8fd0d6af1bfc2
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
-/
import Mathlib.CategoryTheory.Closed.Monoidal
import Mathlib.Algebra.Category.ModuleCat.Monoidal.Symmetric
+#align_import algebra.category.Module.monoidal.closed from "leanprover-community/mathlib"@"74403a3b2551b0970855e14ef5e8fd0d6af1bfc2"
+
/-!
# The monoidal closed structure on `Module R`.
-/
@@ -62,6 +62,8 @@ theorem ihom_map_apply {M N P : ModuleCat.{u} R} (f : N ⟶ P) (g : ModuleCat.of
set_option linter.uppercaseLean3 false in
#align Module.ihom_map_apply ModuleCat.ihom_map_apply
+open MonoidalCategory
+
-- porting note: `CoeFun` was replaced by `FunLike`
-- I can't seem to express the function coercion here without writing `@FunLike.coe`.
@[simp]
The unported dependencies are