src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy
changeset 67399 eab6ce8368fa
parent 67226 ec32cdaab97b
equal deleted inserted replaced
67398:5eb932e604a2 67399:eab6ce8368fa
   329   qed
   329   qed
   330 qed
   330 qed
   331 
   331 
   332 subsection \<open>Preprocessor Inlining\<close>
   332 subsection \<open>Preprocessor Inlining\<close>
   333 
   333 
   334 definition "equals == (op =)"
   334 definition "equals == (=)"
   335  
   335  
   336 inductive zerozero' :: "nat * nat => bool" where
   336 inductive zerozero' :: "nat * nat => bool" where
   337   "equals (x, y) (0, 0) ==> zerozero' (x, y)"
   337   "equals (x, y) (0, 0) ==> zerozero' (x, y)"
   338 
   338 
   339 code_pred (expected_modes: i => bool) zerozero' .
   339 code_pred (expected_modes: i => bool) zerozero' .