mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 16:21:46 +03:00
16 lines
295 B
Idris
16 lines
295 B
Idris
|
module Data.List.Algebra
|
||
|
|
||
|
import Control.Algebra
|
||
|
import Data.List
|
||
|
|
||
|
%default total
|
||
|
|
||
|
public export
|
||
|
SemigroupV (List ty) where
|
||
|
semigroupOpIsAssociative = appendAssociative
|
||
|
|
||
|
public export
|
||
|
MonoidV (List ty) where
|
||
|
monoidNeutralIsNeutralL = appendNilRightNeutral
|
||
|
monoidNeutralIsNeutralR _ = Refl
|