tuned comments;
authorwenzelm
Wed, 29 Dec 2010 12:22:38 +0100
changeset 41408 08a072ca6348
parent 41407 2878845bc549
child 41409 0bc364f772ef
tuned comments;
src/HOL/Mutabelle/mutabelle.ML
src/HOL/Mutabelle/mutabelle_extra.ML
--- 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 ();
 
--- a/src/HOL/Mutabelle/mutabelle_extra.ML	Wed Dec 29 12:16:49 2010 +0100
+++ b/src/HOL/Mutabelle/mutabelle_extra.ML	Wed Dec 29 12:22:38 2010 +0100
@@ -1,8 +1,9 @@
 (*  Title:      HOL/Mutabelle/mutabelle_extra.ML
     Author:     Stefan Berghofer, Jasmin Blanchette, Lukas Bulwahn, TU Muenchen
 
-    Invokation of Counterexample generators
+Invokation of Counterexample generators.
 *)
+
 signature MUTABELLE_EXTRA =
 sig