Nominal/FSet.thy
changeset 2249 1476c26d4310
parent 2238 8ddf1330f2ed
child 2250 c3fd4e42bb4a
equal deleted inserted replaced
2246:8f493d371234 2249:1476c26d4310
  1660 
  1660 
  1661 lemma "(\<lambda> (c::'s \<Rightarrow> bool). \<exists>(x::'s). c = rel x) = {c. \<exists>x. c = rel x}"
  1661 lemma "(\<lambda> (c::'s \<Rightarrow> bool). \<exists>(x::'s). c = rel x) = {c. \<exists>x. c = rel x}"
  1662 apply(auto simp add: mem_def)
  1662 apply(auto simp add: mem_def)
  1663 done
  1663 done
  1664 
  1664 
       
  1665 lemma ball_reg_right_unfolded: "(\<forall>x. R x \<longrightarrow> P x \<longrightarrow> Q x) \<longrightarrow> (All P \<longrightarrow> Ball R Q)"
       
  1666 apply rule
       
  1667 apply (rule ball_reg_right)
       
  1668 apply auto
       
  1669 done
  1665 
  1670 
  1666 end
  1671 end