src/HOL/Tools/inductive_set.ML
changeset 49324 4f28543ae7fa
parent 49170 03bee3a6a1b7
child 50774 ac53370dfae1
--- a/src/HOL/Tools/inductive_set.ML	Wed Sep 12 13:56:49 2012 +0200
+++ b/src/HOL/Tools/inductive_set.ML	Wed Sep 12 14:46:13 2012 +0200
@@ -21,7 +21,7 @@
     (binding * string option * mixfix) list ->
     (binding * string option * mixfix) list ->
     (Attrib.binding * string) list -> (Facts.ref * Attrib.src list) list ->
-    bool -> local_theory -> Inductive.inductive_result * local_theory
+    local_theory -> Inductive.inductive_result * local_theory
   val mono_add: attribute
   val mono_del: attribute
   val codegen_preproc: theory -> thm list -> thm list
@@ -574,11 +574,11 @@
 val ind_set_decl = Inductive.gen_ind_decl add_ind_set_def;
 
 val _ =
-  Outer_Syntax.local_theory' @{command_spec "inductive_set"} "define inductive sets"
+  Outer_Syntax.local_theory @{command_spec "inductive_set"} "define inductive sets"
     (ind_set_decl false);
 
 val _ =
-  Outer_Syntax.local_theory' @{command_spec "coinductive_set"} "define coinductive sets"
+  Outer_Syntax.local_theory @{command_spec "coinductive_set"} "define coinductive sets"
     (ind_set_decl true);
 
 end;