author | huffman |
Thu, 26 Feb 2009 08:48:33 -0800 | |
changeset 30130 | e23770bc97c8 |
parent 29759 | bcb79ddf57da |
child 30270 | 61811c9224a6 |
permissions | -rw-r--r-- |
theory Isar imports Base begin chapter {* Isar language elements *} text {* The primary Isar language consists of three main categories of language elements: \begin{enumerate} \item Proof commands \item Proof methods \item Attributes \end{enumerate} *} section {* Proof commands *} text FIXME section {* Proof methods *} text FIXME section {* Attributes *} text FIXME end