Zulip Chat Archive

Stream: new members

Topic: natural composition


Nicolas Rolland (Aug 18 2023 at 21:02):

mathematical composition of function is defined

@[inline] def Function.comp {α : Sort u} {β : Sort v} {δ : Sort w} (f : β  δ) (g : α  β) : α  δ :=
  fun x => f (g x)

Is there a natural composition operator which goes the other way ?

Sky Wilshaw (Aug 19 2023 at 20:01):

Consider the notation |>: https://leanprover-community.github.io/mathlib4_docs/Init/Notation.html#%C2%ABterm_|%3E_%C2%BB (doesn't answer the question)

Jireh Loreaux (Aug 20 2023 at 02:30):

There is in category theory.


Last updated: Dec 20 2023 at 11:08 UTC