src/HOL/Predicate_Compile_Examples/Hotel_Example.thy
changeset 38734 e5508a74b11f
parent 38733 4b8fd91ea59a
child 38949 1afa9e89c885
--- a/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Wed Aug 25 16:59:51 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Wed Aug 25 16:59:53 2010 +0200
@@ -69,7 +69,7 @@
 | "hotel (e # s) = (hotel s & (case e of
   Check_in g r (k,k') \<Rightarrow> k = currk s r \<and> k' \<notin> issued s |
   Enter g r (k,k') \<Rightarrow> (k,k') : cards s g & (roomk s r : {k, k'}) |
-  Exit g r \<Rightarrow> False))"
+  Exit g r \<Rightarrow> g : isin s r))"
 
 lemma issued_nil: "issued [] = {Key0}"
 by (auto simp add: initk_def)
@@ -86,7 +86,7 @@
 
 ML {* Code_Prolog.options := {ensure_groundness = true} *}
 
-values 10 "{s. hotel s}"
+values 40 "{s. hotel s}"
 
 
 setup {* Quickcheck.add_generator ("prolog", Code_Prolog.quickcheck) *}