src/HOL/Extraction.thy
changeset 24194 96013f81faef
parent 24162 8dfd5dd65d82
child 25424 170f4cc34697
--- a/src/HOL/Extraction.thy	Thu Aug 09 15:52:38 2007 +0200
+++ b/src/HOL/Extraction.thy	Thu Aug 09 15:52:42 2007 +0200
@@ -6,7 +6,7 @@
 header {* Program extraction for HOL *}
 
 theory Extraction
-imports Datatype Option
+imports Datatype
 uses "Tools/rewrite_hol_proof.ML"
 begin