src/HOL/ex/CTL.thy
changeset 32587 caa5ada96a00
parent 26813 6a4d5ca6d2e5
child 32960 69916a850301
equal deleted inserted replaced
32584:89b1f0cd9180 32587:caa5ada96a00
    93     fix x assume l: "x \<in> lfp f"
    93     fix x assume l: "x \<in> lfp f"
    94     show "x \<in> - gfp (\<lambda>s. - f (- s))"
    94     show "x \<in> - gfp (\<lambda>s. - f (- s))"
    95     proof
    95     proof
    96       assume "x \<in> gfp (\<lambda>s. - f (- s))"
    96       assume "x \<in> gfp (\<lambda>s. - f (- s))"
    97       then obtain u where "x \<in> u" and "u \<subseteq> - f (- u)"
    97       then obtain u where "x \<in> u" and "u \<subseteq> - f (- u)"
    98 	by (auto simp add: gfp_def Sup_set_eq)
    98         by (auto simp add: gfp_def)
    99       then have "f (- u) \<subseteq> - u" by auto
    99       then have "f (- u) \<subseteq> - u" by auto
   100       then have "lfp f \<subseteq> - u" by (rule lfp_lowerbound)
   100       then have "lfp f \<subseteq> - u" by (rule lfp_lowerbound)
   101       from l and this have "x \<notin> u" by auto
   101       from l and this have "x \<notin> u" by auto
   102       with `x \<in> u` show False by contradiction
   102       with `x \<in> u` show False by contradiction
   103     qed
   103     qed