src/HOL/Imperative_HOL/ex/Linked_Lists.thy
changeset 58889 5b7a9633cfa8
parent 58333 ec949d7206bb
child 61076 bdc1e2f0a86a
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (*  Title:      HOL/Imperative_HOL/ex/Linked_Lists.thy
     1 (*  Title:      HOL/Imperative_HOL/ex/Linked_Lists.thy
     2     Author:     Lukas Bulwahn, TU Muenchen
     2     Author:     Lukas Bulwahn, TU Muenchen
     3 *)
     3 *)
     4 
     4 
     5 header {* Linked Lists by ML references *}
     5 section {* Linked Lists by ML references *}
     6 
     6 
     7 theory Linked_Lists
     7 theory Linked_Lists
     8 imports "../Imperative_HOL" "~~/src/HOL/Library/Code_Target_Int"
     8 imports "../Imperative_HOL" "~~/src/HOL/Library/Code_Target_Int"
     9 begin
     9 begin
    10 
    10