src/HOL/HOL.thy
changeset 30980 fe0855471964
parent 30970 3fe2e418a071
child 31024 0fdf666e08bf
equal deleted inserted replaced
30979:10eb446df3c7 30980:fe0855471964
     6 
     6 
     7 theory HOL
     7 theory HOL
     8 imports Pure "~~/src/Tools/Code_Generator"
     8 imports Pure "~~/src/Tools/Code_Generator"
     9 uses
     9 uses
    10   ("Tools/hologic.ML")
    10   ("Tools/hologic.ML")
       
    11   "~~/src/Tools/auto_solve.ML"
    11   "~~/src/Tools/IsaPlanner/zipper.ML"
    12   "~~/src/Tools/IsaPlanner/zipper.ML"
    12   "~~/src/Tools/IsaPlanner/isand.ML"
    13   "~~/src/Tools/IsaPlanner/isand.ML"
    13   "~~/src/Tools/IsaPlanner/rw_tools.ML"
    14   "~~/src/Tools/IsaPlanner/rw_tools.ML"
    14   "~~/src/Tools/IsaPlanner/rw_inst.ML"
    15   "~~/src/Tools/IsaPlanner/rw_inst.ML"
    15   "~~/src/Tools/intuitionistic.ML"
    16   "~~/src/Tools/intuitionistic.ML"
  1919 *}
  1920 *}
  1920 
  1921 
  1921 quickcheck_params [size = 5, iterations = 50]
  1922 quickcheck_params [size = 5, iterations = 50]
  1922 
  1923 
  1923 
  1924 
  1924 subsection {* Nitpick hooks *}
  1925 subsection {* Nitpick setup *}
  1925 
  1926 
  1926 text {* This will be relocated once Nitpick is moved to HOL. *}
  1927 text {* This will be relocated once Nitpick is moved to HOL. *}
  1927 
  1928 
  1928 ML {*
  1929 ML {*
  1929 structure Nitpick_Const_Def_Thms = NamedThmsFun
  1930 structure Nitpick_Const_Def_Thms = NamedThmsFun
  1945 (
  1946 (
  1946   val name = "nitpick_ind_intro"
  1947   val name = "nitpick_ind_intro"
  1947   val description = "introduction rules for (co)inductive predicates as needed by Nitpick"
  1948   val description = "introduction rules for (co)inductive predicates as needed by Nitpick"
  1948 )
  1949 )
  1949 *}
  1950 *}
  1950 setup {* Nitpick_Const_Def_Thms.setup
  1951 
  1951          #> Nitpick_Const_Simp_Thms.setup
  1952 setup {*
  1952          #> Nitpick_Const_Psimp_Thms.setup
  1953   Nitpick_Const_Def_Thms.setup
  1953          #> Nitpick_Ind_Intro_Thms.setup *}
  1954   #> Nitpick_Const_Simp_Thms.setup
       
  1955   #> Nitpick_Const_Psimp_Thms.setup
       
  1956   #> Nitpick_Ind_Intro_Thms.setup
       
  1957 *}
       
  1958 
  1954 
  1959 
  1955 subsection {* Legacy tactics and ML bindings *}
  1960 subsection {* Legacy tactics and ML bindings *}
  1956 
  1961 
  1957 ML {*
  1962 ML {*
  1958 fun strip_tac i = REPEAT (resolve_tac [impI, allI] i);
  1963 fun strip_tac i = REPEAT (resolve_tac [impI, allI] i);