src/HOL/Quickcheck_Narrowing.thy
changeset 69605 a96320074298
parent 69593 3dda49e08b9d
child 69690 1fb204399d8d
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
   190 hide_type (open) cfun
   190 hide_type (open) cfun
   191 hide_const (open) Constant eval_cfun Abs_cfun Rep_cfun
   191 hide_const (open) Constant eval_cfun Abs_cfun Rep_cfun
   192 
   192 
   193 subsubsection \<open>Setting up the counterexample generator\<close>
   193 subsubsection \<open>Setting up the counterexample generator\<close>
   194 
   194 
   195 external_file "~~/src/HOL/Tools/Quickcheck/Narrowing_Engine.hs"
   195 external_file \<open>~~/src/HOL/Tools/Quickcheck/Narrowing_Engine.hs\<close>
   196 external_file "~~/src/HOL/Tools/Quickcheck/PNF_Narrowing_Engine.hs"
   196 external_file \<open>~~/src/HOL/Tools/Quickcheck/PNF_Narrowing_Engine.hs\<close>
   197 ML_file "Tools/Quickcheck/narrowing_generators.ML"
   197 ML_file \<open>Tools/Quickcheck/narrowing_generators.ML\<close>
   198 
   198 
   199 definition narrowing_dummy_partial_term_of :: "('a :: partial_term_of) itself => narrowing_term => term"
   199 definition narrowing_dummy_partial_term_of :: "('a :: partial_term_of) itself => narrowing_term => term"
   200 where
   200 where
   201   "narrowing_dummy_partial_term_of = partial_term_of"
   201   "narrowing_dummy_partial_term_of = partial_term_of"
   202 
   202 
   316            (Generated'_Code.Const \"Groups.uminus'_class.uminus\" (mkFunT t t))
   316            (Generated'_Code.Const \"Groups.uminus'_class.uminus\" (mkFunT t t))
   317            (mkNumber (- i)); } in mkNumber)"
   317            (mkNumber (- i)); } in mkNumber)"
   318 
   318 
   319 subsection \<open>The \<open>find_unused_assms\<close> command\<close>
   319 subsection \<open>The \<open>find_unused_assms\<close> command\<close>
   320 
   320 
   321 ML_file "Tools/Quickcheck/find_unused_assms.ML"
   321 ML_file \<open>Tools/Quickcheck/find_unused_assms.ML\<close>
   322 
   322 
   323 subsection \<open>Closing up\<close>
   323 subsection \<open>Closing up\<close>
   324 
   324 
   325 hide_type narrowing_type narrowing_term narrowing_cons property
   325 hide_type narrowing_type narrowing_term narrowing_cons property
   326 hide_const map_cons nth error toEnum marker empty Narrowing_cons conv non_empty ensure_testable all exists drawn_from around_zero
   326 hide_const map_cons nth error toEnum marker empty Narrowing_cons conv non_empty ensure_testable all exists drawn_from around_zero