src/Doc/IsarRef/HOL_Specific.thy
changeset 52476 7d7b4e285ea7
parent 52435 6646bb548c6b
child 52637 1501ebe39711
equal deleted inserted replaced
52475:445ae7a4e4e1 52476:7d7b4e285ea7
  2457   \item @{command (HOL) "code_identifier"} associates a a series of symbols
  2457   \item @{command (HOL) "code_identifier"} associates a a series of symbols
  2458   (constants, type constructors, classes, class relations, instances,
  2458   (constants, type constructors, classes, class relations, instances,
  2459   module names) with target-specific hints how these symbols shall be named.
  2459   module names) with target-specific hints how these symbols shall be named.
  2460   \emph{Warning:} These hints are still subject to name disambiguation.
  2460   \emph{Warning:} These hints are still subject to name disambiguation.
  2461   @{command (HOL) "code_modulename"} is a legacy variant for
  2461   @{command (HOL) "code_modulename"} is a legacy variant for
  2462   @{command (HOL) "code_identifier"} on module names.
  2462   @{command (HOL) "code_identifier"} on module names.  It is at the discretion
       
  2463   of the user to ensure that name prefixes of identifiers in compound
       
  2464   statements like type classes or datatypes are still the same.
  2463 
  2465 
  2464   \item @{command (HOL) "code_reflect"} without a ``@{text "file"}''
  2466   \item @{command (HOL) "code_reflect"} without a ``@{text "file"}''
  2465   argument compiles code into the system runtime environment and
  2467   argument compiles code into the system runtime environment and
  2466   modifies the code generator setup that future invocations of system
  2468   modifies the code generator setup that future invocations of system
  2467   runtime code generation referring to one of the ``@{text
  2469   runtime code generation referring to one of the ``@{text