src/HOL/ex/Predicate_Compile_ex.thy
changeset 33104 560372b461e5
parent 32673 d5db9cf85401
child 33105 1e4146bf841c
equal deleted inserted replaced
32949:aa6c470a962a 33104:560372b461e5
   359 "w \<in> A\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b] + 1"
   359 "w \<in> A\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b] + 1"
   360 "w \<in> B\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = b] = length [x \<leftarrow> w. x = a] + 1"
   360 "w \<in> B\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = b] = length [x \<leftarrow> w. x = a] + 1"
   361 (*quickcheck[generator = pred_compile, size=5, iterations=1]*)
   361 (*quickcheck[generator = pred_compile, size=5, iterations=1]*)
   362 oops
   362 oops
   363 
   363 
   364 
       
   365 section {* Lambda *}
   364 section {* Lambda *}
       
   365 
   366 datatype type =
   366 datatype type =
   367     Atom nat
   367     Atom nat
   368   | Fun type type    (infixr "\<Rightarrow>" 200)
   368   | Fun type type    (infixr "\<Rightarrow>" 200)
   369 
   369 
   370 datatype dB =
   370 datatype dB =