made SML/NJ happy
authorLars Hupel <lars.hupel@mytum.de>
Wed, 05 Feb 2014 15:44:32 +0100
changeset 55335 8192d3acadbe
parent 55334 5f5104069b33
child 55336 1401434a7e83
made SML/NJ happy
src/Pure/Tools/simplifier_trace.ML
--- a/src/Pure/Tools/simplifier_trace.ML	Wed Feb 05 11:47:56 2014 +0100
+++ b/src/Pure/Tools/simplifier_trace.ML	Wed Feb 05 15:44:32 2014 +0100
@@ -48,15 +48,15 @@
      breakpoints = empty_breakpoints}
   val extend = I
   fun merge ({max_depth = max_depth1, mode = mode1, interactive = interactive1,
-              breakpoints = breakpoints1, ...},
+              breakpoints = breakpoints1, ...}: T,
              {max_depth = max_depth2, mode = mode2, interactive = interactive2,
-              breakpoints = breakpoints2, ...}) =
+              breakpoints = breakpoints2, ...}: T) =
     {max_depth = Int.max (max_depth1, max_depth2),
      depth = 0,
      mode = merge_modes mode1 mode2,
      interactive = interactive1 orelse interactive2,
      parent = 0,
-     breakpoints = merge_breakpoints (breakpoints1, breakpoints2)}
+     breakpoints = merge_breakpoints (breakpoints1, breakpoints2)}: T
 )
 
 fun map_breakpoints f_term f_thm =
@@ -191,7 +191,9 @@
   end
 
 
-fun step {term, thm, unconditional, ctxt, rrule} =
+type data = {term: term, thm: thm, unconditional: bool, ctxt: Proof.context, rrule: rrule}
+
+fun step ({term, thm, unconditional, ctxt, rrule}: data) =
   let
     val (matching_terms, thm_triggered) = is_breakpoint (term, rrule) (Context.Proof ctxt)
 
@@ -292,7 +294,7 @@
           (output_result res; put (#1 res))
   in Context.the_proof context' end
 
-fun indicate_failure {term, ctxt, thm, rrule, ...} ctxt' =
+fun indicate_failure ({term, ctxt, thm, rrule, ...}: data) ctxt' =
   let
     fun payload () =
       let