src/HOL/HOL.thy
changeset 39039 bef9e5dd0fd0
parent 39033 e8b68ec3bb9c
parent 39036 dff91b90d74c
child 39159 0dec18004e75
--- a/src/HOL/HOL.thy	Thu Sep 02 12:30:22 2010 +0200
+++ b/src/HOL/HOL.thy	Thu Sep 02 13:45:39 2010 +0200
@@ -32,6 +32,7 @@
   ("Tools/recfun_codegen.ML")
   "Tools/async_manager.ML"
   "Tools/try.ML"
+  ("Tools/cnf_funcs.ML")
 begin
 
 setup {* Intuitionistic.method_setup @{binding iprover} *}
@@ -1645,7 +1646,6 @@
   "(\<not> \<not>(P)) = P"
 by blast+
 
-
 subsection {* Basic ML bindings *}
 
 ML {*
@@ -1699,6 +1699,7 @@
 val trans = @{thm trans}
 *}
 
+use "Tools/cnf_funcs.ML"
 
 subsection {* Code generator setup *}