src/HOL/Library/State_Monad.thy
changeset 27368 9f90ac19e32b
parent 26588 d83271bfaba5
child 27487 c8a6ce181805
equal deleted inserted replaced
27367:a75d71c73362 27368:9f90ac19e32b
     4 *)
     4 *)
     5 
     5 
     6 header {* Combinators syntax for generic, open state monads (single threaded monads) *}
     6 header {* Combinators syntax for generic, open state monads (single threaded monads) *}
     7 
     7 
     8 theory State_Monad
     8 theory State_Monad
     9 imports List
     9 imports Plain List
    10 begin
    10 begin
    11 
    11 
    12 subsection {* Motivation *}
    12 subsection {* Motivation *}
    13 
    13 
    14 text {*
    14 text {*