src/HOL/Relation.thy
changeset 64633 5ebcf6c525f1
parent 64632 9df24b8b6c0a
child 64634 5bd30359e46e
equal deleted inserted replaced
64632:9df24b8b6c0a 64633:5ebcf6c525f1
  1147   using assms
  1147   using assms
  1148   by (induct R)
  1148   by (induct R)
  1149     (auto simp: comp_fun_commute.fold_insert comp_fun_commute_relcomp_fold insert_relcomp_fold
  1149     (auto simp: comp_fun_commute.fold_insert comp_fun_commute_relcomp_fold insert_relcomp_fold
  1150       cong: if_cong)
  1150       cong: if_cong)
  1151 
  1151 
  1152 text \<open>Misc\<close>
       
  1153 
       
  1154 abbreviation (input) transP :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> bool"
       
  1155   where "transP r \<equiv> trans {(x, y). r x y}"  (* FIXME drop *)
       
  1156 
       
  1157 end
  1152 end