diff agda/deltaM.agda @ 90:55d11ce7e223

Unify levels on data type. only use suc to proofs
author Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp>
date Mon, 19 Jan 2015 12:11:38 +0900
parents 5411ce26d525
children bcd4fe52a504
line wrap: on
line diff
--- a/agda/deltaM.agda	Mon Jan 19 11:48:41 2015 +0900
+++ b/agda/deltaM.agda	Mon Jan 19 12:11:38 2015 +0900
@@ -54,11 +54,11 @@
 checkOut (S n) (deltaM (mono x))    = x
 checkOut {l} {A} {M} {functorM} {monadM} (S n) (deltaM (delta _ d)) = checkOut {l} {A} {M} {functorM} {monadM} n (deltaM d)
 
-{-
-deltaM-fmap : {l ll : Level} {A : Set l} {B : Set ll} 
-           {M : {l' : Level} -> Set l' -> Set l'}
-           {functorM : {l' : Level} -> Functor {l'} M}
-           {monadM : {l' : Level} {A : Set l'} -> Monad {l'} {A} M functorM}
-           -> (A -> B) -> DeltaM M {functorM} {monadM} A -> DeltaM M {functorM} {monadM} B
-deltaM-fmap {l} {ll} {A} {B} {M} {functorM} f (deltaM d) = deltaM (Functor.fmap delta-is-functor (Functor.fmap functorM f) d)
--}
\ No newline at end of file
+
+open Functor
+deltaM-fmap : {l : Level} {A B : Set l}
+              {M : {l' : Level} -> Set l' -> Set l'}
+              {functorM : {l' : Level} -> Functor {l'} M}
+              {monadM : {l' : Level} {A : Set l'} -> Monad {l'} {A} M functorM}
+              -> (A -> B) -> DeltaM M {functorM} {monadM} A -> DeltaM M {functorM} {monadM} B
+deltaM-fmap {l} {A} {B} {M} {functorM} f (deltaM d) = deltaM (fmap delta-is-functor (fmap functorM f) d)