src/Doc/Implementation/Local_Theory.thy
changeset 61439 2bf52eec4e8a
parent 58618 782f0b662cae
child 61458 987533262fc2
--- a/src/Doc/Implementation/Local_Theory.thy	Wed Oct 14 15:06:42 2015 +0200
+++ b/src/Doc/Implementation/Local_Theory.thy	Wed Oct 14 15:10:32 2015 +0200
@@ -105,7 +105,7 @@
 
   \begin{description}
 
-  \item Type @{ML_type local_theory} represents local theories.
+  \<^descr> Type @{ML_type local_theory} represents local theories.
   Although this is merely an alias for @{ML_type Proof.context}, it is
   semantically a subtype of the same: a @{ML_type local_theory} holds
   target information as special context data.  Subtyping means that
@@ -113,7 +113,7 @@
   with operations on expecting a regular @{text "ctxt:"}~@{ML_type
   Proof.context}.
 
-  \item @{ML Named_Target.init}~@{text "before_exit name thy"}
+  \<^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
   non-empty name refers to a @{command locale} or @{command class}
@@ -121,7 +121,7 @@
   useful for experimentation --- normally the Isar toplevel already
   takes care to initialize the local theory context.
 
-  \item @{ML Local_Theory.define}~@{text "((b, mx), (a, rhs))
+  \<^descr> @{ML Local_Theory.define}~@{text "((b, mx), (a, rhs))
   lthy"} defines a local entity according to the specification that is
   given relatively to the current @{text "lthy"} context.  In
   particular the term of the RHS may refer to earlier local entities
@@ -141,7 +141,7 @@
   declarations such as @{attribute simp}, while non-trivial rules like
   @{attribute simplified} are better avoided.
 
-  \item @{ML Local_Theory.note}~@{text "(a, ths) lthy"} is
+  \<^descr> @{ML Local_Theory.note}~@{text "(a, ths) lthy"} is
   analogous to @{ML Local_Theory.define}, but defines facts instead of
   terms.  There is also a slightly more general variant @{ML
   Local_Theory.notes} that defines several facts (with attribute