src/HOL/ex/ATP_Export.thy
changeset 43468 c768f7adb711
parent 43400 3d03f4472883
--- a/src/HOL/ex/ATP_Export.thy	Sun Jun 19 18:12:49 2011 +0200
+++ b/src/HOL/ex/ATP_Export.thy	Sun Jun 19 18:12:49 2011 +0200
@@ -4,7 +4,7 @@
 begin
 
 ML {*
-val do_it = false; (* switch to "true" to generate files *)
+val do_it = false; (* switch to "true" to generate the files *)
 val thy = @{theory Complex_Main};
 val ctxt = @{context}
 *}