src/HOL/HOL.thy
changeset 32668 b2de45007537
parent 32661 f4d179d91af2
child 32733 71618deaf777
equal deleted inserted replaced
32667:09546e654222 32668:b2de45007537
  2021 
  2021 
  2022 quickcheck_params [size = 5, iterations = 50]
  2022 quickcheck_params [size = 5, iterations = 50]
  2023 
  2023 
  2024 subsection {* Preprocessing for the predicate compiler *}
  2024 subsection {* Preprocessing for the predicate compiler *}
  2025 
  2025 
  2026 setup {* Predicate_Compile_Preproc_Const_Defs.setup *}
  2026 ML {*
       
  2027 structure Predicate_Compile_Alternative_Defs = Named_Thms
       
  2028 (
       
  2029   val name = "code_pred_def"
       
  2030   val description = "alternative definitions of constants for the Predicate Compiler"
       
  2031 )
       
  2032 *}
       
  2033 
       
  2034 ML {*
       
  2035 structure Predicate_Compile_Inline_Defs = Named_Thms
       
  2036 (
       
  2037   val name = "code_pred_inline"
       
  2038   val description = "inlining definitions for the Predicate Compiler"
       
  2039 )
       
  2040 *}
       
  2041 
       
  2042 setup {*
       
  2043   Predicate_Compile_Alternative_Defs.setup
       
  2044   #> Predicate_Compile_Inline_Defs.setup
       
  2045   #> Predicate_Compile_Preproc_Const_Defs.setup
       
  2046 *}
  2027 
  2047 
  2028 subsection {* Nitpick setup *}
  2048 subsection {* Nitpick setup *}
  2029 
  2049 
  2030 text {* This will be relocated once Nitpick is moved to HOL. *}
  2050 text {* This will be relocated once Nitpick is moved to HOL. *}
  2031 
  2051