Skip to content

Commit

Permalink
chore(category_theory/closed/monoidal): correct error in doc string (#…
Browse files Browse the repository at this point in the history
…13385)

Sorry, should have done this immediately when @b-mehta pointed out my mistake.



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Apr 12, 2022
1 parent ef8e256 commit 73ec5b2
Showing 1 changed file with 4 additions and 6 deletions.
10 changes: 4 additions & 6 deletions src/category_theory/closed/monoidal.lean
Expand Up @@ -23,6 +23,10 @@ namespace category_theory
open category monoidal_category

/-- An object `X` is (right) closed if `(X ⊗ -)` is a left adjoint. -/
-- Note that this class carries a particular choice of right adjoint,
-- (which is only unique up to isomorphism),
-- not merely the existence of such, and
-- so definitional properties of instances may be important.
class closed {C : Type u} [category.{v} C] [monoidal_category.{v} C] (X : C) :=
(is_adj : is_left_adjoint (tensor_left X))

Expand Down Expand Up @@ -71,12 +75,6 @@ variables [closed A]

/--
This is the internal hom `A ⟶[C] -`.
Note that this is essentially an opaque definition,
and so will not agree definitionally with any "native" internal hom the category has.
TODO: we could introduce a `has_ihom` class
that allows specifying a particular definition of the internal hom,
and provide a low priority opaque instance.
-/
def ihom : C ⥤ C :=
(@closed.is_adj _ _ _ A _).right
Expand Down

0 comments on commit 73ec5b2

Please sign in to comment.