src/HOL/Hoare/SepLogHeap.thy
changeset 42174 d0be2722ce9f
parent 41959 b460124855b8
child 44890 22f665a2e91c
equal deleted inserted replaced
42173:5d33c12ccf22 42174:d0be2722ce9f
     8 
     8 
     9 theory SepLogHeap
     9 theory SepLogHeap
    10 imports Main
    10 imports Main
    11 begin
    11 begin
    12 
    12 
    13 types heap = "(nat \<Rightarrow> nat option)"
    13 type_synonym heap = "(nat \<Rightarrow> nat option)"
    14 
    14 
    15 text{* @{text "Some"} means allocated, @{text "None"} means
    15 text{* @{text "Some"} means allocated, @{text "None"} means
    16 free. Address @{text "0"} serves as the null reference. *}
    16 free. Address @{text "0"} serves as the null reference. *}
    17 
    17 
    18 subsection "Paths in the heap"
    18 subsection "Paths in the heap"