Zulip Chat Archive
Stream: Is there code for X?
Topic: exponential object
Chris Henson (Aug 29 2024 at 03:01):
I'm a bit confused about some of the category theory typeclasses. For example I'm not sure how to finish this:
import Mathlib.CategoryTheory.Closed.Cartesian
open CategoryTheory
def eval {X : Type} [Category X] [Limits.HasFiniteProducts X] [CartesianClosed X] (a b : X) : a ⨯ (a ⟹ b) ⟶ b := by
sorry
Kim Morrison (Aug 29 2024 at 03:50):
def eval {X : Type} [Category X] [Limits.HasFiniteProducts X] [CartesianClosed X] (a b : X) :
a ⨯ (a ⟹ b) ⟶ b := (exp.ev a).app b
Kim Morrison (Aug 29 2024 at 03:50):
That whole file is a bit more "point free" than it really needs to be. :-)
Chris Henson (Aug 29 2024 at 03:57):
Great, thank you!
Last updated: May 02 2025 at 03:31 UTC