doc-src/IsarImplementation/Thy/ML.thy
changeset 21502 7f3ea2b3bab6
parent 21148 3a64d58a9f49
child 22293 3593a76c9ed3
--- a/doc-src/IsarImplementation/Thy/ML.thy	Thu Nov 23 20:33:42 2006 +0100
+++ b/doc-src/IsarImplementation/Thy/ML.thy	Thu Nov 23 20:34:21 2006 +0100
@@ -5,6 +5,8 @@
 
 chapter {* Aesthetics of ML programming *}
 
+text FIXME
+
 text {* This style guide is loosely based on
   \url{http://caml.inria.fr/resources/doc/guides/guidelines.en.html}.
 %  FIMXE \url{http://www.cs.cornell.edu/Courses/cs312/2003sp/handouts/style.htm}
@@ -85,7 +87,7 @@
       while keeping its length to the absolutely neccessary minimum.
       Always give the same name to function arguments which
       have the same meaning. Separate words by underscores
-      (``{\ttfamily int\_of\_string}'', not ``{\ttfamily intOfString}'')
+      (``@{verbatim int_of_string}'', not ``@{verbatim intOfString}'')
 
   \end{description}
 *}