src/HOL/ex/Bit_Lists.thy
changeset 72515 c7038c397ae3
parent 72262 a282abb07642
child 74097 6d7be1227d02
--- a/src/HOL/ex/Bit_Lists.thy	Thu Oct 29 09:59:40 2020 +0000
+++ b/src/HOL/ex/Bit_Lists.thy	Thu Oct 29 10:03:03 2020 +0000
@@ -5,7 +5,7 @@
 
 theory Bit_Lists
   imports
-    "HOL-Word.Word" "HOL-Library.More_List"
+    "HOL-Library.Word" "HOL-Library.More_List"
 begin
 
 subsection \<open>Fragments of algebraic bit representations\<close>