| changeset 15131 | c69542757a4d |
| parent 14981 | e73f8140af78 |
| child 15140 | 322485b816ac |
--- a/src/HOL/Extraction.thy Mon Aug 16 14:21:54 2004 +0200 +++ b/src/HOL/Extraction.thy Mon Aug 16 14:22:27 2004 +0200 @@ -5,9 +5,10 @@ header {* Program extraction for HOL *} -theory Extraction = Datatype -files - "Tools/rewrite_hol_proof.ML": +theory Extraction +import Datatype +files "Tools/rewrite_hol_proof.ML" +begin subsection {* Setup *}