src/FOL/FOL.thy
changeset 24830 a7b3ab44d993
parent 24097 86734ba03ca2
child 26286 3ff5d257f175
--- a/src/FOL/FOL.thy	Thu Oct 04 14:42:11 2007 +0200
+++ b/src/FOL/FOL.thy	Thu Oct 04 14:42:47 2007 +0200
@@ -11,6 +11,7 @@
   "~~/src/Provers/classical.ML"
   "~~/src/Provers/blast.ML"
   "~~/src/Provers/clasimp.ML"
+  "~~/src/Tools/induct.ML"
   ("cladata.ML")
   ("blastdata.ML")
   ("simpdata.ML")
@@ -74,7 +75,7 @@
   apply (erule r1)
   done
 
-lemmas case_split = case_split_thm [case_names True False, cases type: o]
+lemmas case_split = case_split_thm [case_names True False]
 
 (*HOL's more natural case analysis tactic*)
 ML {*
@@ -273,15 +274,16 @@
 text {* Method setup. *}
 
 ML {*
-  structure InductMethod = InductMethodFun
-  (struct
+  structure Induct = InductFun
+  (
     val cases_default = @{thm case_split}
     val atomize = @{thms induct_atomize}
     val rulify = @{thms induct_rulify}
     val rulify_fallback = @{thms induct_rulify_fallback}
-  end);
+  );
 *}
 
-setup InductMethod.setup
+setup Induct.setup
+declare case_split [cases type: o]
 
 end