src/HOL/Tools/Sledgehammer/sledgehammer_preplay.ML
changeset 54504 096f7d452164
parent 53761 4d34e267fba9
child 54700 64177ce0a7bd
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_preplay.ML	Tue Nov 19 18:34:04 2013 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_preplay.ML	Tue Nov 19 18:38:25 2013 +0100
@@ -35,7 +35,7 @@
   val proof_preplay_interface :
     bool -> Proof.context -> string -> string -> bool -> Time.time
     -> isar_proof -> preplay_interface
-end
+end;
 
 structure Sledgehammer_Preplay : SLEDGEHAMMER_PREPLAY =
 struct
@@ -312,4 +312,4 @@
         overall_preplay_stats = overall_preplay_stats}
     end
 
-end
+end;