src/Doc/Locales/Examples.thy
changeset 58620 7435b6a3f72e
parent 51799 8fcf6e32544e
child 61419 3c3f8b182e4b
equal deleted inserted replaced
58619:4b41df5fef81 58620:7435b6a3f72e
   293 text {* The syntax of the locale commands discussed in this tutorial is
   293 text {* The syntax of the locale commands discussed in this tutorial is
   294   shown in Table~\ref{tab:commands}.  The grammar is complete with the
   294   shown in Table~\ref{tab:commands}.  The grammar is complete with the
   295   exception of the context elements \isakeyword{constrains} and
   295   exception of the context elements \isakeyword{constrains} and
   296   \isakeyword{defines}, which are provided for backward
   296   \isakeyword{defines}, which are provided for backward
   297   compatibility.  See the Isabelle/Isar Reference
   297   compatibility.  See the Isabelle/Isar Reference
   298   Manual~\cite{IsarRef} for full documentation.  *}
   298   Manual @{cite IsarRef} for full documentation.  *}
   299 
   299 
   300 
   300 
   301 section {* Import \label{sec:import} *}
   301 section {* Import \label{sec:import} *}
   302 
   302 
   303 text {* 
   303 text {* 
   761   stored, and conclusions that will be
   761   stored, and conclusions that will be
   762   added to $l_2$ in future are automatically propagated to $l_1$.
   762   added to $l_2$ in future are automatically propagated to $l_1$.
   763   The sublocale relation is transitive --- that is, propagation takes
   763   The sublocale relation is transitive --- that is, propagation takes
   764   effect along chains of sublocales.  Even cycles in the sublocale relation are
   764   effect along chains of sublocales.  Even cycles in the sublocale relation are
   765   supported, as long as these cycles do not lead to infinite chains.
   765   supported, as long as these cycles do not lead to infinite chains.
   766   Details are discussed in the technical report \cite{Ballarin2006a}.
   766   Details are discussed in the technical report @{cite Ballarin2006a}.
   767   See also Section~\ref{sec:infinite-chains} of this tutorial.  *}
   767   See also Section~\ref{sec:infinite-chains} of this tutorial.  *}
   768 
   768 
   769 end
   769 end