doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 29560 fa6c5d62adf5
parent 29114 715178f6ae31
child 30169 9531eaafd781
child 30240 5b25fee0362c
equal deleted inserted replaced
29559:fe9cfe076c23 29560:fa6c5d62adf5
     1 (* $Id$ *)
       
     2 
       
     3 theory HOL_Specific
     1 theory HOL_Specific
     4 imports Main
     2 imports Main
     5 begin
     3 begin
     6 
     4 
     7 chapter {* Isabelle/HOL \label{ch:hol} *}
     5 chapter {* Isabelle/HOL \label{ch:hol} *}
  1161 
  1159 
  1162   \item @{command (HOL) "code_modulename"} declares aliasings from one
  1160   \item @{command (HOL) "code_modulename"} declares aliasings from one
  1163   module name onto another.
  1161   module name onto another.
  1164 
  1162 
  1165   \item @{command (HOL) "code_abort"} declares constants which are not
  1163   \item @{command (HOL) "code_abort"} declares constants which are not
  1166   required to have a definition by means of defining equations; if
  1164   required to have a definition by means of code equations; if
  1167   needed these are implemented by program abort instead.
  1165   needed these are implemented by program abort instead.
  1168 
  1166 
  1169   \item @{attribute (HOL) code} explicitly selects (or with option
  1167   \item @{attribute (HOL) code} explicitly selects (or with option
  1170   ``@{text "del"}'' deselects) a defining equation for code
  1168   ``@{text "del"}'' deselects) a code equation for code
  1171   generation.  Usually packages introducing defining equations provide
  1169   generation.  Usually packages introducing code equations provide
  1172   a reasonable default setup for selection.
  1170   a reasonable default setup for selection.
  1173 
  1171 
  1174   \item @{attribute (HOL) code}~@{text inline} declares (or with
  1172   \item @{attribute (HOL) code}~@{text inline} declares (or with
  1175   option ``@{text "del"}'' removes) inlining theorems which are
  1173   option ``@{text "del"}'' removes) inlining theorems which are
  1176   applied as rewrite rules to any defining equation during
  1174   applied as rewrite rules to any code equation during
  1177   preprocessing.
  1175   preprocessing.
  1178 
  1176 
  1179   \item @{command (HOL) "print_codesetup"} gives an overview on
  1177   \item @{command (HOL) "print_codesetup"} gives an overview on
  1180   selected defining equations, code generator datatypes and
  1178   selected code equations, code generator datatypes and
  1181   preprocessor setup.
  1179   preprocessor setup.
  1182 
  1180 
  1183   \end{description}
  1181   \end{description}
  1184 *}
  1182 *}
  1185 
  1183