src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML
changeset 52374 ddb16589b711
parent 52369 0b395800fdf0
child 52453 2cba5906d836
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Thu Jun 13 14:35:05 2013 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Thu Jun 13 16:58:20 2013 -0400
@@ -5,7 +5,7 @@
 Isar proof reconstruction from ATP proofs.
 *)
 
-signature SLEDGEHAMMER_PROOF_RECONSTRUCT =
+signature SLEDGEHAMMER_RECONSTRUCT =
 sig
   type 'a proof = 'a ATP_Proof.proof
   type stature = ATP_Problem_Generate.stature
@@ -45,7 +45,7 @@
     -> string
 end;
 
-structure Sledgehammer_Reconstruct : SLEDGEHAMMER_PROOF_RECONSTRUCT =
+structure Sledgehammer_Reconstruct : SLEDGEHAMMER_RECONSTRUCT =
 struct
 
 open ATP_Util