src/Doc/Codegen/Further.thy
changeset 52378 08dbf9ff2140
parent 51717 9e7d1c139569
child 52665 5f817bad850a
equal deleted inserted replaced
52377:afa72aaed518 52378:08dbf9ff2140
   122   A solution is to declare module names explicitly.  Let use assume
   122   A solution is to declare module names explicitly.  Let use assume
   123   the three cyclically dependent modules are named \emph{A}, \emph{B}
   123   the three cyclically dependent modules are named \emph{A}, \emph{B}
   124   and \emph{C}.  Then, by stating
   124   and \emph{C}.  Then, by stating
   125 *}
   125 *}
   126 
   126 
   127 code_modulename %quote SML
   127 code_identifier %quote
   128   A ABC
   128   code_module A \<rightharpoonup> (SML) ABC
   129   B ABC
   129 | code_module B \<rightharpoonup> (SML) ABC
   130   C ABC
   130 | code_module C \<rightharpoonup> (SML) ABC
   131 
   131 
   132 text {*
   132 text {*
   133   \noindent we explicitly map all those modules on \emph{ABC},
   133   \noindent we explicitly map all those modules on \emph{ABC},
   134   resulting in an ad-hoc merge of this three modules at serialisation
   134   resulting in an ad-hoc merge of this three modules at serialisation
   135   time.
   135   time.