src/HOL/Imperative_HOL/Heap_Monad.thy
changeset 41413 64cd30d6b0b8
parent 40671 5e46057ba8e0
child 42949 618adb3584e5
equal deleted inserted replaced
41412:35f30e07fe0d 41413:64cd30d6b0b8
     3 *)
     3 *)
     4 
     4 
     5 header {* A monad with a polymorphic heap and primitive reasoning infrastructure *}
     5 header {* A monad with a polymorphic heap and primitive reasoning infrastructure *}
     6 
     6 
     7 theory Heap_Monad
     7 theory Heap_Monad
     8 imports Heap Monad_Syntax Code_Natural
     8 imports
       
     9   Heap
       
    10   "~~/src/HOL/Library/Monad_Syntax"
       
    11   "~~/src/HOL/Library/Code_Natural"
     9 begin
    12 begin
    10 
    13 
    11 subsection {* The monad *}
    14 subsection {* The monad *}
    12 
    15 
    13 subsubsection {* Monad construction *}
    16 subsubsection {* Monad construction *}