diff -r 1884c40f1539 -r e467ae7aa808 src/Doc/Implementation/Local_Theory.thy --- a/src/Doc/Implementation/Local_Theory.thy Sun Oct 18 21:30:01 2015 +0200 +++ b/src/Doc/Implementation/Local_Theory.thy Sun Oct 18 22:57:09 2015 +0200 @@ -5,12 +5,12 @@ chapter \Local theory specifications \label{ch:local-theory}\ text \ - A \emph{local theory} combines aspects of both theory and proof + 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 assumptions. A local theory is represented as a regular proof - context, augmented by administrative data about the \emph{target - context}. + context, augmented by administrative data about the \<^emph>\target + context\. The target is usually derived from the background theory by adding local @{text "\"} and @{text "\"} elements, plus @@ -45,7 +45,7 @@ \secref{sec:variables}). These definitional primitives essentially act like @{text "let"}-bindings within a local context that may already contain earlier @{text "let"}-bindings and some initial - @{text "\"}-bindings. Thus we gain \emph{dependent definitions} + @{text "\"}-bindings. Thus we gain \<^emph>\dependent definitions\ that are relative to an initial axiomatic context. The following diagram illustrates this idea of axiomatic elements versus definitional elements: @@ -72,7 +72,7 @@ The cumulative sequence of @{text "\"} and @{text "\"} produced at package runtime is managed by the local theory - infrastructure by means of an \emph{auxiliary context}. Thus the + infrastructure by means of an \<^emph>\auxiliary context\. Thus the system holds up the impression of working within a fully abstract situation with hypothetical entities: @{text "\ c \ t"} always results in a literal fact @{text "\<^BG>c \ t\<^EN>"}, where @@ -113,7 +113,7 @@ \<^descr> @{ML Named_Target.init}~@{text "before_exit name thy"} initializes a local theory derived from the given background theory. - An empty name refers to a \emph{global theory} context, and a + An empty name refers to a \<^emph>\global theory\ context, and a non-empty name refers to a @{command locale} or @{command class} context (a fully-qualified internal name is expected here). This is useful for experimentation --- normally the Isar toplevel already @@ -132,7 +132,7 @@ Unless an explicit name binding is given for the RHS, the resulting fact will be called @{text "b_def"}. Any given attributes are applied to that same fact --- immediately in the auxiliary context - \emph{and} in any transformed versions stemming from target-specific + \<^emph>\and\ in any transformed versions stemming from target-specific policies or any later interpretations of results from the target context (think of @{command locale} and @{command interpretation}, for example). This means that attributes should be usually plain