tuned;
authorwenzelm
Mon, 18 Apr 2016 14:26:42 +0200
changeset 63010 8e0378864478
parent 63009 3c2df99b7b1d
child 63011 301e631666a0
tuned;
src/HOL/Tools/Function/function_common.ML
--- a/src/HOL/Tools/Function/function_common.ML	Mon Apr 18 14:26:21 2016 +0200
+++ b/src/HOL/Tools/Function/function_common.ML	Mon Apr 18 14:26:42 2016 +0200
@@ -69,7 +69,7 @@
     domintros: bool,
     partials: bool}
   type preproc = function_config -> Proof.context -> fixes -> term spec ->
-    (term list * (thm list -> thm spec) * (thm list -> thm list list) * string list)
+    term list * (thm list -> thm spec) * (thm list -> thm list list) * string list
   val fname_of : term -> string
   val mk_case_names : int -> string -> int -> string list
   val empty_preproc : (Proof.context -> ((string * typ) * mixfix) list -> term list -> 'c) ->
@@ -209,7 +209,7 @@
   partials: bool}
 
 type preproc = function_config -> Proof.context -> fixes -> term spec ->
-  (term list * (thm list -> thm spec) * (thm list -> thm list list) * string list)
+  term list * (thm list -> thm spec) * (thm list -> thm list list) * string list
 
 val fname_of = fst o dest_Free o fst o strip_comb o fst o HOLogic.dest_eq o
   HOLogic.dest_Trueprop o Logic.strip_imp_concl o snd o dest_all_all