src/HOL/Extraction.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15393 2e6a9146caca
--- a/src/HOL/Extraction.thy	Tue Aug 17 11:00:24 2004 +0200
+++ b/src/HOL/Extraction.thy	Wed Aug 18 11:09:40 2004 +0200
@@ -6,7 +6,7 @@
 header {* Program extraction for HOL *}
 
 theory Extraction
-import Datatype
+imports Datatype
 files "Tools/rewrite_hol_proof.ML"
 begin