Idris2/libs/contrib/Control/Algebra/Implementations.idr
2020-07-17 08:25:20 -05:00

22 lines
403 B
Idris

module Control.Algebra.Implementations
import Control.Algebra
-- This file is for algebra implementations with nowhere else to go.
%default total
-- Functions ---------------------------
Semigroup (ty -> ty) where
(<+>) = (.)
SemigroupV (ty -> ty) where
semigroupOpIsAssociative _ _ _ = Refl
Monoid (ty -> ty) where
neutral = id
MonoidV (ty -> ty) where
monoidNeutralIsNeutralR _ = Refl