src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy
changeset 39648 655307cb8489
parent 39545 631cf48c7894
child 39654 1207e39f0c7f
--- a/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy	Thu Sep 23 10:39:25 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy	Thu Sep 23 14:50:13 2010 +0200
@@ -522,7 +522,6 @@
 thm filter2.equation
 thm filter2.random_dseq_equation
 
-(*
 inductive filter3
 for P
 where
@@ -530,9 +529,9 @@
 
 code_pred (expected_modes: (o => bool) => i => o => bool, (o => bool) => i => i => bool , (i => bool) => i => o => bool, (i => bool) => i => i => bool) [skip_proof] filter3 .
 
-code_pred [dseq] filter3 .
-thm filter3.dseq_equation
-*)
+code_pred filter3 .
+thm filter3.equation
+
 (*
 inductive filter4
 where