doc-src/IsarAdvanced/Codegen/Thy/Codegen.thy
changeset 21222 6dfdb69e83ef
parent 21217 0425fc57510f
child 21223 b3bdc1abc7d3
equal deleted inserted replaced
21221:ef30d1e6f03a 21222:6dfdb69e83ef
   423 
   423 
   424   \begin{itemize}
   424   \begin{itemize}
   425 
   425 
   426   \item the Isabelle/Isar Reference Manual \cite{isabelle-isar-ref}
   426   \item the Isabelle/Isar Reference Manual \cite{isabelle-isar-ref}
   427     for exhaustive syntax diagrams.
   427     for exhaustive syntax diagrams.
   428   \item or \fixme{ref} which deals with foundational issues
   428   \item or \fixme[ref] which deals with foundational issues
   429     of the code generator framework.
   429     of the code generator framework.
   430 
   430 
   431   \end{itemize}
   431   \end{itemize}
   432 *}
   432 *}
   433 
   433 
  1369   \begin{warn}
  1369   \begin{warn}
  1370     Some interfaces discussed here have not reached
  1370     Some interfaces discussed here have not reached
  1371     a final state yet.
  1371     a final state yet.
  1372     Changes likely to occur in future.
  1372     Changes likely to occur in future.
  1373   \end{warn}
  1373   \end{warn}
       
  1374 
       
  1375   \fixme
  1374 *}
  1376 *}
  1375 
  1377 
  1376 subsubsection {* Data depending on the theory's executable content *}
  1378 subsubsection {* Data depending on the theory's executable content *}
  1377 
  1379 
  1378 text {*
  1380 text {*
  1441   @{index_ML DatatypeCodegen.add_codetypes_hook_bootstrap: "
  1443   @{index_ML DatatypeCodegen.add_codetypes_hook_bootstrap: "
  1442       DatatypeCodegen.hook -> theory -> theory"}
  1444       DatatypeCodegen.hook -> theory -> theory"}
  1443   \end{mldecls}
  1445   \end{mldecls}
  1444 *}
  1446 *}
  1445 
  1447 
  1446 (*text {*
  1448 text {*
  1447   \emph{Happy proving, happy hacking!}
  1449   \fixme
  1448 *}*)
  1450 %  \emph{Happy proving, happy hacking!}
       
  1451 *}
  1449 
  1452 
  1450 end
  1453 end