ProgTutorial/Package/Ind_Interface.thy
changeset 365 718beb785213
parent 346 0fea8b7a14a1
child 426 d94755882e36
--- a/ProgTutorial/Package/Ind_Interface.thy	Fri Oct 30 09:42:16 2009 +0100
+++ b/ProgTutorial/Package/Ind_Interface.thy	Fri Oct 30 09:42:16 2009 +0100
@@ -129,7 +129,7 @@
 *}
 (*<*)ML %no{*fun add_inductive_cmd pred_specs rule_specs lthy = lthy 
    fun add_inductive pred_specs rule_specs lthy = lthy*}(*>*)
-ML_val %linenosgray{*val specification =
+ML_val %linenosgray{*val specification : (local_theory -> local_theory) parser =
   spec_parser >>
     (fn (pred_specs, rule_specs) => add_inductive_cmd pred_specs rule_specs)