src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy
changeset 47433 07f4bf913230
parent 47108 2a1953f0d20d
child 51143 0a2371e7ced3
equal deleted inserted replaced
47306:56d72c923281 47433:07f4bf913230
  1025   (o * o => bool) => i * o => bool,
  1025   (o * o => bool) => i * o => bool,
  1026   (o * o => bool) => o * i => bool,
  1026   (o * o => bool) => o * i => bool,
  1027   (o * o => bool) => i * i => bool) [inductify] converse .
  1027   (o * o => bool) => i * i => bool) [inductify] converse .
  1028 
  1028 
  1029 thm converse.equation
  1029 thm converse.equation
  1030 code_pred [inductify] rel_comp .
  1030 code_pred [inductify] relcomp .
  1031 thm rel_comp.equation
  1031 thm relcomp.equation
  1032 code_pred [inductify] Image .
  1032 code_pred [inductify] Image .
  1033 thm Image.equation
  1033 thm Image.equation
  1034 declare singleton_iff[code_pred_inline]
  1034 declare singleton_iff[code_pred_inline]
  1035 declare Id_on_def[unfolded Bex_def UNION_eq singleton_iff, code_pred_def]
  1035 declare Id_on_def[unfolded Bex_def UNION_eq singleton_iff, code_pred_def]
  1036 
  1036