mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-18 00:31:57 +03:00
16 lines
334 B
Idris
16 lines
334 B
Idris
|
module Data.Morphisms.Algebra
|
||
|
|
||
|
import Control.Algebra
|
||
|
import Data.Morphisms
|
||
|
|
||
|
%default total
|
||
|
|
||
|
public export
|
||
|
SemigroupV (Endomorphism ty) where
|
||
|
semigroupOpIsAssociative (Endo _) (Endo _) (Endo _) = Refl
|
||
|
|
||
|
public export
|
||
|
MonoidV (Endomorphism ty) where
|
||
|
monoidNeutralIsNeutralL (Endo _) = Refl
|
||
|
monoidNeutralIsNeutralR (Endo _) = Refl
|