src/HOL/Imperative_HOL/Heap.thy
changeset 66453 cc19f7ca2ed6
parent 66004 797ef4889177
child 67443 3abf6a722518
--- a/src/HOL/Imperative_HOL/Heap.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Imperative_HOL/Heap.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -5,7 +5,7 @@
 section \<open>A polymorphic heap based on cantor encodings\<close>
 
 theory Heap
-imports Main "~~/src/HOL/Library/Countable"
+imports Main "HOL-Library.Countable"
 begin
 
 subsection \<open>Representable types\<close>