src/Pure/type.ML
changeset 2979 db6941221197
parent 2964 557a11310988
child 2991 d9f6299dbf9f
--- a/src/Pure/type.ML	Thu Apr 17 18:45:43 1997 +0200
+++ b/src/Pure/type.ML	Thu Apr 17 18:46:58 1997 +0200
@@ -65,8 +65,9 @@
   val get_sort: type_sig -> (indexname -> sort option) -> (indexname * sort) list
     -> indexname -> sort
   val constrain: term -> typ -> term
-  val infer_types: type_sig * (string -> typ option) * (indexname -> typ option)
-    * (indexname -> sort option) * string list * bool * typ list * term list
+  val infer_types: (term -> Pretty.T) -> (typ -> Pretty.T)
+    -> type_sig -> (string -> typ option) -> (indexname -> typ option)
+    -> (indexname -> sort option) -> string list -> bool -> typ list -> term list
     -> term list * (indexname * typ) list
 end;
 
@@ -871,14 +872,14 @@
     "?" :: _ => true
   | _ => false);
 
-fun infer_types (tsig, const_type, def_type, def_sort, used, freeze, pat_Ts, raw_ts) =
+fun infer_types prt prT tsig const_type def_type def_sort used freeze pat_Ts raw_ts =
   let
     val TySg {classrel, arities, ...} = tsig;
     val pat_Ts' = map (cert_typ tsig) pat_Ts;
     val raw_ts' =
       map (decode_types tsig (is_some o const_type) def_type def_sort) raw_ts;
     val (ts, Ts, unifier) =
-      TypeInfer.infer_types const_type classrel arities used freeze
+      TypeInfer.infer_types prt prT const_type classrel arities used freeze
         q_is_param raw_ts' pat_Ts';
   in
     (ts, unifier)