diff -r 4f169d2cf6f3 -r 782f0b662cae src/Doc/Implementation/Local_Theory.thy --- a/src/Doc/Implementation/Local_Theory.thy Tue Oct 07 21:28:24 2014 +0200 +++ b/src/Doc/Implementation/Local_Theory.thy Tue Oct 07 21:29:59 2014 +0200 @@ -2,9 +2,9 @@ imports Base begin -chapter {* Local theory specifications \label{ch:local-theory} *} +chapter \Local theory specifications \label{ch:local-theory}\ -text {* +text \ A \emph{local theory} combines aspects of both theory and proof context (cf.\ \secref{sec:context}), such that definitional specifications may be given relatively to parameters and @@ -33,12 +33,12 @@ Isabelle. Although a few old packages only work for global theories, the standard way of implementing definitional packages in Isabelle is via the local theory interface. -*} +\ -section {* Definitional elements *} +section \Definitional elements\ -text {* +text \ There are separate elements @{text "\ c \ t"} for terms, and @{text "\ b = thm"} for theorems. Types are treated implicitly, according to Hindley-Milner discipline (cf.\ @@ -91,9 +91,9 @@ terms and theorems that stem from the hypothetical @{text "\"} and @{text "\"} elements, transformed by the particular target policy (see @{cite \\S4--5\ "Haftmann-Wenzel:2009"} - for details). *} + for details).\ -text %mlref {* +text %mlref \ \begin{mldecls} @{index_ML_type local_theory: Proof.context} \\ @{index_ML Named_Target.init: "string -> theory -> local_theory"} \\[1ex] @@ -151,15 +151,15 @@ command, or @{command declare} if an empty name binding is given. \end{description} -*} +\ -section {* Morphisms and declarations \label{sec:morphisms} *} +section \Morphisms and declarations \label{sec:morphisms}\ -text {* +text \ %FIXME See also @{cite "Chaieb-Wenzel:2007"}. -*} +\ end