src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy
changeset 38728 182b180e9804
parent 38727 c7f5f0b7dc7f
child 38731 2c8a595af43e
equal deleted inserted replaced
38727:c7f5f0b7dc7f 38728:182b180e9804
   185 
   185 
   186 ML {* Code_Prolog.options := {ensure_groundness = true} *}
   186 ML {* Code_Prolog.options := {ensure_groundness = true} *}
   187 
   187 
   188 values 2 "{y. notB y}"
   188 values 2 "{y. notB y}"
   189 
   189 
       
   190 inductive notAB :: "abc * abc \<Rightarrow> bool"
       
   191 where
       
   192   "y \<noteq> A \<Longrightarrow> z \<noteq> B \<Longrightarrow> notAB (y, z)"
       
   193 
       
   194 code_pred notAB .
       
   195 
       
   196 values 5 "{y. notAB y}"
       
   197 
   190 end
   198 end