src/HOL/Quickcheck_Examples/Hotel_Example.thy
changeset 48255 968602739b54
parent 48222 fcca68383808
child 51143 0a2371e7ced3
equal deleted inserted replaced
48254:63e0ca00b952 48255:968602739b54
   188   "hotel s ==> feels_safe s r ==> g \<in> isin s r ==> owns s r = Some g"
   188   "hotel s ==> feels_safe s r ==> g \<in> isin s r ==> owns s r = Some g"
   189 (* quickcheck[exhaustive, size = 9, timeout = 2000] -- maybe possible with a lot of time *)
   189 (* quickcheck[exhaustive, size = 9, timeout = 2000] -- maybe possible with a lot of time *)
   190 quickcheck[narrowing, size = 7, expect = counterexample]
   190 quickcheck[narrowing, size = 7, expect = counterexample]
   191 oops
   191 oops
   192 
   192 
   193 ebd
   193 end