src/HOL/Tools/Function/fun.ML
changeset 58826 2ed2eaabe3df
parent 56254 a2dd9200854d
child 59159 9312710451f5
--- a/src/HOL/Tools/Function/fun.ML	Wed Oct 29 17:01:44 2014 +0100
+++ b/src/HOL/Tools/Function/fun.ML	Wed Oct 29 19:01:49 2014 +0100
@@ -14,8 +14,6 @@
   val add_fun_cmd : (binding * string option * mixfix) list ->
     (Attrib.binding * string) list -> Function_Common.function_config ->
     bool -> local_theory -> Proof.context
-
-  val setup : theory -> theory
 end
 
 structure Function_Fun : FUNCTION_FUN =
@@ -148,8 +146,8 @@
   else
     Function_Common.empty_preproc check_defs config ctxt fixes spec
 
-val setup =
-  Context.theory_map (Function_Common.set_preproc sequential_preproc)
+val _ = Theory.setup (Context.theory_map (Function_Common.set_preproc sequential_preproc))
+
 
 
 val fun_config = FunctionConfig { sequential=true, default=NONE,