mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-21 02:31:50 +03:00
19 lines
482 B
Idris
19 lines
482 B
Idris
module Control.Monad.Algebra
|
|
|
|
import Control.Algebra
|
|
import Control.Monad.Identity
|
|
|
|
%default total
|
|
|
|
public export
|
|
SemigroupV ty => SemigroupV (Identity ty) where
|
|
semigroupOpIsAssociative (Id l) (Id c) (Id r) =
|
|
rewrite semigroupOpIsAssociative l c r in Refl
|
|
|
|
public export
|
|
MonoidV ty => MonoidV (Identity ty) where
|
|
monoidNeutralIsNeutralL (Id l) =
|
|
rewrite monoidNeutralIsNeutralL l in Refl
|
|
monoidNeutralIsNeutralR (Id r) =
|
|
rewrite monoidNeutralIsNeutralR r in Refl
|