src/HOL/Imperative_HOL/ex/Linked_Lists.thy
changeset 48430 6cbfe187a0f9
parent 44890 22f665a2e91c
child 50630 1ea90e8046dc
--- a/src/HOL/Imperative_HOL/ex/Linked_Lists.thy	Sun Jul 22 23:36:11 2012 +0200
+++ b/src/HOL/Imperative_HOL/ex/Linked_Lists.thy	Mon Jul 23 09:26:55 2012 +0200
@@ -5,7 +5,7 @@
 header {* Linked Lists by ML references *}
 
 theory Linked_Lists
-imports "../Imperative_HOL" Code_Integer
+imports "../Imperative_HOL" "~~/src/HOL/Library/Code_Integer"
 begin
 
 section {* Definition of Linked Lists *}
@@ -1003,3 +1003,4 @@
 export_code test_1 test_2 test_3 checking SML SML_imp OCaml? OCaml_imp? Haskell? Scala? Scala_imp?
 
 end
+