src/HOL/Mutabelle/mutabelle.ML
changeset 41408 08a072ca6348
parent 41067 c78a2d402736
child 41755 404d94506599
--- a/src/HOL/Mutabelle/mutabelle.ML	Wed Dec 29 12:16:49 2010 +0100
+++ b/src/HOL/Mutabelle/mutabelle.ML	Wed Dec 29 12:22:38 2010 +0100
@@ -1,8 +1,9 @@
 (*  Title:      HOL/Mutabelle/mutabelle.ML
     Author:     Veronika Ortner, TU Muenchen
 
-    Mutation of theorems
+Mutation of theorems.
 *)
+
 signature MUTABELLE =
 sig
  val testgen_name : string Unsynchronized.ref
@@ -80,13 +81,10 @@
  end;
 
 
-(*helper function in order to properly print a term*)
+(*possibility to print a given term for debugging purposes*)
 
 fun prt x = Pretty.writeln (Syntax.pretty_term_global @{theory Main} x);
 
-
-(*possibility to print a given term for debugging purposes*)
-
 val debug = (Unsynchronized.ref false);
 fun debug_msg mutterm = if (!debug) then (prt mutterm) else ();