src/HOL/Library/Countable.thy
changeset 27487 c8a6ce181805
parent 27368 9f90ac19e32b
child 28823 dcbef866c9e2
--- a/src/HOL/Library/Countable.thy	Fri Jul 04 16:33:08 2008 +0200
+++ b/src/HOL/Library/Countable.thy	Mon Jul 07 08:47:17 2008 +0200
@@ -6,7 +6,7 @@
 header {* Encoding (almost) everything into natural numbers *}
 
 theory Countable
-imports Plain List Hilbert_Choice
+imports Plain "~~/src/HOL/List" "~~/src/HOL/Hilbert_Choice"
 begin
 
 subsection {* The class of countable types *}