Idris2/libs/contrib/Control/Algebra/Implementations.idr

22 lines
403 B
Idris
Raw Normal View History

2020-07-14 01:52:22 +03:00
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