removed unused signature
authorboehmes
Wed, 02 Sep 2009 16:02:37 +0200
changeset 32495 6decc1ffdbed
parent 32490 6a48db3e627c
child 32496 4ab00a2642c3
removed unused signature
src/HOL/Tools/Mirabelle/Tools/mirabelle.ML
--- a/src/HOL/Tools/Mirabelle/Tools/mirabelle.ML	Wed Sep 02 14:11:45 2009 +0200
+++ b/src/HOL/Tools/Mirabelle/Tools/mirabelle.ML	Wed Sep 02 16:02:37 2009 +0200
@@ -4,14 +4,20 @@
 
 signature MIRABELLE =
 sig
-  type action
-  val register : string * action -> theory -> theory
-
+  (* configuration *)
   val logfile : string Config.T
   val timeout : int Config.T
   val start_line : int Config.T
   val end_line : int Config.T
+  val setup : theory -> theory
 
+  (* core *)
+  type action
+  val register : string * action -> theory -> theory
+  val step_hook : Toplevel.transition -> Toplevel.state -> Toplevel.state ->
+    unit
+
+  (* utility functions *)
   val goal_thm_of : Proof.state -> thm
   val can_apply : Time.time -> (Proof.context -> int -> tactic) ->
     Proof.state -> bool
@@ -23,19 +29,20 @@
 
 
 
-signature MIRABELLE_EXT =
-sig
-  include MIRABELLE
-  val setup : theory -> theory
-  val step_hook : Toplevel.transition -> Toplevel.state -> Toplevel.state ->
-    unit
-end
+structure Mirabelle : MIRABELLE_EXT =
+struct
+
+(* Mirabelle configuration *)
+
+val (logfile, setup1) = Attrib.config_string "mirabelle_logfile" ""
+val (timeout, setup2) = Attrib.config_int "mirabelle_timeout" 30
+val (start_line, setup3) = Attrib.config_int "mirabelle_start_line" 0
+val (end_line, setup4) = Attrib.config_int "mirabelle_end_line" ~1
+
+val setup = setup1 #> setup2 #> setup3 #> setup4
 
 
 
-structure Mirabelle : MIRABELLE_EXT =
-struct
-
 (* Mirabelle core *)
 
 type action = {pre: Proof.state, post: Toplevel.state option,
@@ -52,13 +59,6 @@
 
 val register = Actions.map o Symtab.update_new
 
-val (logfile, setup1) = Attrib.config_string "mirabelle_logfile" ""
-val (timeout, setup2) = Attrib.config_int "mirabelle_timeout" 30
-val (start_line, setup3) = Attrib.config_int "mirabelle_start_line" 0
-val (end_line, setup4) = Attrib.config_int "mirabelle_end_line" ~1
-
-val setup = setup1 #> setup2 #> setup3 #> setup4
-
 local
 
 fun log thy s =