src/HOL/Library/Char_nat.thy
changeset 27368 9f90ac19e32b
parent 26152 cf2cccf17d6d
child 27487 c8a6ce181805
--- a/src/HOL/Library/Char_nat.thy	Thu Jun 26 10:06:54 2008 +0200
+++ b/src/HOL/Library/Char_nat.thy	Thu Jun 26 10:07:01 2008 +0200
@@ -6,7 +6,7 @@
 header {* Mapping between characters and natural numbers *}
 
 theory Char_nat
-imports List
+imports Plain List
 begin
 
 text {* Conversions between nibbles and natural numbers in [0..15]. *}