src/HOL/Predicate_Compile_Examples/Hotel_Example.thy
changeset 38731 2c8a595af43e
parent 38730 5bbdd9a9df62
child 38733 4b8fd91ea59a
--- a/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Wed Aug 25 16:59:49 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Wed Aug 25 16:59:50 2010 +0200
@@ -84,10 +84,10 @@
 lemma [code_pred_inline]: "(op -) == (%A B x. A x \<and> \<not> B x)"
 by (auto simp add: Diff_iff[unfolded mem_def] expand_fun_eq intro!: eq_reflection)
 
-code_pred [new_random_dseq inductify, skip_proof] hotel .
-
 ML {* Code_Prolog.options := {ensure_groundness = true} *}
 
 values 10 "{s. hotel s}"
 
+
+
 end
\ No newline at end of file