src/HOL/Quickcheck_Examples/Hotel_Example.thy
changeset 51143 0a2371e7ced3
parent 48255 968602739b54
child 51272 9c8d63b4b6be
--- a/src/HOL/Quickcheck_Examples/Hotel_Example.thy	Fri Feb 15 08:31:30 2013 +0100
+++ b/src/HOL/Quickcheck_Examples/Hotel_Example.thy	Fri Feb 15 08:31:31 2013 +0100
@@ -105,8 +105,8 @@
   [code]: "cps_of_set (set xs) f = find_first f xs"
 sorry
 
-consts pos_cps_of_set :: "'a set => ('a => (bool * term list) option) => code_numeral => (bool * term list) option"
-consts neg_cps_of_set :: "'a set => ('a Quickcheck_Exhaustive.unknown => term list Quickcheck_Exhaustive.three_valued) => code_numeral => term list Quickcheck_Exhaustive.three_valued"
+consts pos_cps_of_set :: "'a set => ('a => (bool * term list) option) => natural => (bool * term list) option"
+consts neg_cps_of_set :: "'a set => ('a Quickcheck_Exhaustive.unknown => term list Quickcheck_Exhaustive.three_valued) => natural => term list Quickcheck_Exhaustive.three_valued"
 
 lemma
   [code]: "pos_cps_of_set (set xs) f i = find_first f xs"