| author | haftmann |
| Tue, 07 Mar 2006 14:09:48 +0100 | |
| changeset 19202 | 0b9eb4b0ad98 |
| parent 18554 | bff7a1466fe4 |
| child 20489 | a684fc70d04e |
| permissions | -rw-r--r-- |
(* $Id$ *) theory "ML" imports base begin chapter {* Aesthetics of ML programming *} text {* FIXME style guide, see also \url{http://caml.inria.fr/resources/doc/guides/guidelines.en.html} and \url{http://www.cs.cornell.edu/Courses/cs312/2003sp/handouts/style.htm} *} chapter {* Basic library functions *} text {* FIXME beyond the basis library definition *} end