module StateMonad () where import Prelude hiding (return, (>>=)) data ST s a = S (s -> (a, s)) {-@ data ST s a
Bool> = S { x:: (f:s
-> (a, s
)) } @-} {-@ foo :: (Int, {v:Int|v >=0})@-} foo = apply action 0 {-@ action :: ST <{\v -> v>=0 }> Int Int@-} action :: ST Int Int action = act1 `comp` \n1 -> act2 `comp` \n2 -> return n1 {-@ act1 :: ST <{\v -> v>=0 } > Int Int @-} act1 :: ST Int Int act1 = S (\n -> (n, n+1)) act2 :: ST Int Int act2 = S (\n -> (n, n+9)) {-@ apply :: forall
Bool>. ST
s a -> f:s
-> (a, s
) @-}
apply :: ST s a -> s -> (a, s)
apply (S f) x = f x
{-@ return :: forall s {v:a|v=x} @-}
return :: a -> ST s a
return x = S $ \s -> (x, s)
{-@ comp :: forall < p :: s -> Bool>. ST s a -> (a -> ST s b) -> ST s b @-}
comp :: ST s a -> (a -> ST s b) -> ST s b
(S m) `comp` k
= S $ \s -> case (m s) of { (r, new_s) ->
case (k r) of { S k2 ->
(k2 new_s) }}