src/HOL/Quickcheck_Narrowing.thy
changeset 45734 1024dd30da42
parent 45001 5c8d7d6db682
child 45818 53a697f5454a
equal deleted inserted replaced
45733:6bb30ae1abfe 45734:1024dd30da42
   346 primrec eval_cfun :: "'b cfun => 'a => 'b"
   346 primrec eval_cfun :: "'b cfun => 'a => 'b"
   347 where
   347 where
   348   "eval_cfun (Constant c) y = c"
   348   "eval_cfun (Constant c) y = c"
   349 
   349 
   350 hide_type (open) cfun
   350 hide_type (open) cfun
   351 hide_const (open) Constant eval_cfun
   351 hide_const (open) Constant eval_cfun Abs_cfun Rep_cfun
   352 
   352 
   353 subsubsection {* Setting up the counterexample generator *}
   353 subsubsection {* Setting up the counterexample generator *}
   354 
   354 
   355 use "Tools/Quickcheck/narrowing_generators.ML"
   355 use "Tools/Quickcheck/narrowing_generators.ML"
   356 
   356