| author | wenzelm | 
| Mon, 09 Mar 2009 22:43:25 +0100 | |
| changeset 30399 | a4772a650b4e | 
| parent 30272 | 2d612824e642 | 
| child 39842 | 7205191afde4 | 
| 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