made SML/NJ happy
authorsmolkas
Thu, 11 Jul 2013 13:33:20 +0200
changeset 52591 760a567f1609
parent 52590 02713cd2c2cd
child 52592 8a25b17e3d79
child 52593 aedf7b01c6e4
made SML/NJ happy
src/HOL/Tools/Sledgehammer/sledgehammer_compress.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_compress.ML	Thu Jul 11 13:33:19 2013 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_compress.ML	Thu Jul 11 13:33:20 2013 +0200
@@ -119,7 +119,8 @@
 (* PRE CONDITION: the proof must be labeled canocially, see
    Slegehammer_Proof.relabel_proof_canonically *)
 fun compress_proof isar_compress isar_compress_degree merge_timeout_slack
-  { get_time, set_time, preplay_quietly, preplay_fail, ... } proof =
+  ({get_time, set_time, preplay_quietly, preplay_fail, ...} : preplay_interface)
+  proof =
   if isar_compress <= 1.0 then
     proof
   else