src/HOL/ex/Word_Type.thy
changeset 66453 cc19f7ca2ed6
parent 64593 50c715579715
child 66806 a4e82b58d833
--- a/src/HOL/ex/Word_Type.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/ex/Word_Type.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -6,7 +6,7 @@
 theory Word_Type
   imports
     Main
-    "~~/src/HOL/Library/Type_Length"
+    "HOL-Library.Type_Length"
 begin
 
 subsection \<open>Truncating bit representations of numeric types\<close>