author | wenzelm |
Sun, 01 Oct 2006 18:29:26 +0200 | |
changeset 20809 | 6c4fd0b4b63a |
parent 20520 | 05fd007bdeb9 |
child 21148 | 3a64d58a9f49 |
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 NJ basis library proposal *} chapter {* Cookbook *} section {* A method that depends on declarations in the context *} text FIXME end