doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 46028 9f113cdf3d66
parent 45944 e586f6d136b7
child 46280 9be4d8c8d842
child 46447 f37da60a8cc6
equal deleted inserted replaced
46027:ff3c4f2bee01 46028:9f113cdf3d66
  1781     @{command_def (HOL) "code_abort"} & : & @{text "theory \<rightarrow> theory"} \\
  1781     @{command_def (HOL) "code_abort"} & : & @{text "theory \<rightarrow> theory"} \\
  1782     @{command_def (HOL) "code_datatype"} & : & @{text "theory \<rightarrow> theory"} \\
  1782     @{command_def (HOL) "code_datatype"} & : & @{text "theory \<rightarrow> theory"} \\
  1783     @{command_def (HOL) "print_codesetup"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1783     @{command_def (HOL) "print_codesetup"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1784     @{attribute_def (HOL) code_unfold} & : & @{text attribute} \\
  1784     @{attribute_def (HOL) code_unfold} & : & @{text attribute} \\
  1785     @{attribute_def (HOL) code_post} & : & @{text attribute} \\
  1785     @{attribute_def (HOL) code_post} & : & @{text attribute} \\
  1786     @{attribute_def (HOL) code_unfold_post} & : & @{text attribute} \\
  1786     @{attribute_def (HOL) code_abbrev} & : & @{text attribute} \\
  1787     @{command_def (HOL) "print_codeproc"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1787     @{command_def (HOL) "print_codeproc"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1788     @{command_def (HOL) "code_thms"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1788     @{command_def (HOL) "code_thms"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1789     @{command_def (HOL) "code_deps"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1789     @{command_def (HOL) "code_deps"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
  1790     @{command_def (HOL) "code_const"} & : & @{text "theory \<rightarrow> theory"} \\
  1790     @{command_def (HOL) "code_const"} & : & @{text "theory \<rightarrow> theory"} \\
  1791     @{command_def (HOL) "code_type"} & : & @{text "theory \<rightarrow> theory"} \\
  1791     @{command_def (HOL) "code_type"} & : & @{text "theory \<rightarrow> theory"} \\
  1833     ;
  1833     ;
  1834 
  1834 
  1835     @@{attribute (HOL) code_post} ( 'del' ) ?
  1835     @@{attribute (HOL) code_post} ( 'del' ) ?
  1836     ;
  1836     ;
  1837 
  1837 
  1838     @@{attribute (HOL) code_unfold_post}
  1838     @@{attribute (HOL) code_abbrev}
  1839     ;
  1839     ;
  1840 
  1840 
  1841     @@{command (HOL) code_thms} ( constexpr + ) ?
  1841     @@{command (HOL) code_thms} ( constexpr + ) ?
  1842     ;
  1842     ;
  1843 
  1843 
  1938 
  1938 
  1939   \item @{command (HOL) "print_codesetup"} gives an overview on
  1939   \item @{command (HOL) "print_codesetup"} gives an overview on
  1940   selected code equations and code generator datatypes.
  1940   selected code equations and code generator datatypes.
  1941 
  1941 
  1942   \item @{attribute (HOL) code_unfold} declares (or with option
  1942   \item @{attribute (HOL) code_unfold} declares (or with option
  1943   ``@{text "del"}'' removes) theorems which are applied as
  1943   ``@{text "del"}'' removes) theorems which during preprocessing
  1944   rewrite rules to any code equation during preprocessing.
  1944   are applied as rewrite rules to any code equation or evaluation
       
  1945   input.
  1945 
  1946 
  1946   \item @{attribute (HOL) code_post} declares (or with option ``@{text
  1947   \item @{attribute (HOL) code_post} declares (or with option ``@{text
  1947   "del"}'' removes) theorems which are applied as rewrite rules to any
  1948   "del"}'' removes) theorems which are applied as rewrite rules to any
  1948   result of an evaluation.
  1949   result of an evaluation.
  1949 
  1950 
  1950   \item @{attribute (HOL) code_unfold_post} declares equations which are
  1951   \item @{attribute (HOL) code_abbrev} declares equations which are
  1951   applied as rewrite rules to any code equation during preprocessing,
  1952   applied as rewrite rules to any result of an evaluation and
  1952   and symmetrically to any result of an evaluation.
  1953   symmetrically during preprocessing to any code equation or evaluation
  1953   
  1954   input.
       
  1955 
  1954   \item @{command (HOL) "print_codeproc"} prints the setup of the code
  1956   \item @{command (HOL) "print_codeproc"} prints the setup of the code
  1955   generator preprocessor.
  1957   generator preprocessor.
  1956 
  1958 
  1957   \item @{command (HOL) "code_thms"} prints a list of theorems
  1959   \item @{command (HOL) "code_thms"} prints a list of theorems
  1958   representing the corresponding program containing all given
  1960   representing the corresponding program containing all given