| author | berghofe |
| Fri, 07 Apr 2006 11:17:44 +0200 | |
| changeset 19357 | dade85a75c9f |
| parent 18554 | bff7a1466fe4 |
| child 20489 | a684fc70d04e |
| permissions | -rw-r--r-- |
| 18537 | 1 |
|
| 18538 | 2 |
(* $Id$ *) |
3 |
||
4 |
theory "ML" imports base begin |
|
5 |
||
6 |
chapter {* Aesthetics of ML programming *}
|
|
7 |
||
| 18554 | 8 |
text {* FIXME style guide, see also
|
9 |
\url{http://caml.inria.fr/resources/doc/guides/guidelines.en.html} and
|
|
10 |
\url{http://www.cs.cornell.edu/Courses/cs312/2003sp/handouts/style.htm}
|
|
11 |
*} |
|
| 18538 | 12 |
|
13 |
||
14 |
chapter {* Basic library functions *}
|
|
15 |
||
16 |
text {* FIXME beyond the basis library definition *}
|
|
17 |
||
18 |
end |