src/HOL/HOL.thy
changeset 33056 791a4655cae3
parent 33022 c95102496490
child 33084 cd1579e0997a
equal deleted inserted replaced
33055:5a733f325939 33056:791a4655cae3
  2047 subsection {* Nitpick setup *}
  2047 subsection {* Nitpick setup *}
  2048 
  2048 
  2049 text {* This will be relocated once Nitpick is moved to HOL. *}
  2049 text {* This will be relocated once Nitpick is moved to HOL. *}
  2050 
  2050 
  2051 ML {*
  2051 ML {*
  2052 structure Nitpick_Const_Defs = Named_Thms
  2052 structure Nitpick_Defs = Named_Thms
  2053 (
  2053 (
  2054   val name = "nitpick_const_def"
  2054   val name = "nitpick_def"
  2055   val description = "alternative definitions of constants as needed by Nitpick"
  2055   val description = "alternative definitions of constants as needed by Nitpick"
  2056 )
  2056 )
  2057 structure Nitpick_Const_Simps = Named_Thms
  2057 structure Nitpick_Simps = Named_Thms
  2058 (
  2058 (
  2059   val name = "nitpick_const_simp"
  2059   val name = "nitpick_simp"
  2060   val description = "equational specification of constants as needed by Nitpick"
  2060   val description = "equational specification of constants as needed by Nitpick"
  2061 )
  2061 )
  2062 structure Nitpick_Const_Psimps = Named_Thms
  2062 structure Nitpick_Psimps = Named_Thms
  2063 (
  2063 (
  2064   val name = "nitpick_const_psimp"
  2064   val name = "nitpick_psimp"
  2065   val description = "partial equational specification of constants as needed by Nitpick"
  2065   val description = "partial equational specification of constants as needed by Nitpick"
  2066 )
  2066 )
  2067 structure Nitpick_Ind_Intros = Named_Thms
  2067 structure Nitpick_Intros = Named_Thms
  2068 (
  2068 (
  2069   val name = "nitpick_ind_intro"
  2069   val name = "nitpick_intro"
  2070   val description = "introduction rules for (co)inductive predicates as needed by Nitpick"
  2070   val description = "introduction rules for (co)inductive predicates as needed by Nitpick"
  2071 )
  2071 )
  2072 *}
  2072 *}
  2073 
  2073 
  2074 setup {*
  2074 setup {*
  2075   Nitpick_Const_Defs.setup
  2075   Nitpick_Defs.setup
  2076   #> Nitpick_Const_Simps.setup
  2076   #> Nitpick_Simps.setup
  2077   #> Nitpick_Const_Psimps.setup
  2077   #> Nitpick_Psimps.setup
  2078   #> Nitpick_Ind_Intros.setup
  2078   #> Nitpick_Intros.setup
  2079 *}
  2079 *}
  2080 
  2080 
  2081 
  2081 
  2082 subsection {* Legacy tactics and ML bindings *}
  2082 subsection {* Legacy tactics and ML bindings *}
  2083 
  2083