doc-src/IsarAdvanced/Codegen/Thy/ML.thy
changeset 28447 df77ed974a78
parent 28419 f65e8b318581
child 28635 cc53d2ab0170
equal deleted inserted replaced
28446:a01de3b3fa2e 28447:df77ed974a78
   106   Implementing code generator applications on top
   106   Implementing code generator applications on top
   107   of the framework set out so far usually not only
   107   of the framework set out so far usually not only
   108   involves using those primitive interfaces
   108   involves using those primitive interfaces
   109   but also storing code-dependent data and various
   109   but also storing code-dependent data and various
   110   other things.
   110   other things.
   111 
       
   112   \begin{warn}
       
   113     Some interfaces discussed here have not reached
       
   114     a final state yet.
       
   115     Changes likely to occur in future.
       
   116   \end{warn}
       
   117 *}
   111 *}
   118 
   112 
   119 subsubsection {* Data depending on the theory's executable content *}
   113 subsubsection {* Data depending on the theory's executable content *}
   120 
   114 
   121 text {*
   115 text {*
   150     hints that executable content for constants @{text consts}
   144     hints that executable content for constants @{text consts}
   151     has changed.
   145     has changed.
   152 
   146 
   153   \end{description}
   147   \end{description}
   154 
   148 
   155   An instance of @{ML_functor CodeDataFun} provides the following
   149   \noindent An instance of @{ML_functor CodeDataFun} provides the following
   156   interface:
   150   interface:
   157 
   151 
   158   \medskip
   152   \medskip
   159   \begin{tabular}{l}
   153   \begin{tabular}{l}
   160   @{text "get: theory \<rightarrow> T"} \\
   154   @{text "get: theory \<rightarrow> T"} \\
   173 
   167 
   174   \end{description}
   168   \end{description}
   175 *}
   169 *}
   176 
   170 
   177 text {*
   171 text {*
       
   172   \bigskip
       
   173 
   178   \emph{Happy proving, happy hacking!}
   174   \emph{Happy proving, happy hacking!}
   179 *}
   175 *}
   180 
   176 
   181 end
   177 end