src/HOL/MicroJava/DFA/Err.thy
changeset 69597 ff784d5a5bfb
parent 67613 ce654b0e6d69
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   300 apply simp
   300 apply simp
   301 apply fast
   301 apply fast
   302 done 
   302 done 
   303 
   303 
   304 text \<open>
   304 text \<open>
   305   If @{term "AS = {}"} the thm collapses to
   305   If \<^term>\<open>AS = {}\<close> the thm collapses to
   306   @{prop "order r & closed {Err} f & Err +_f Err = Err"}
   306   \<^prop>\<open>order r & closed {Err} f & Err +_f Err = Err\<close>
   307   which may not hold 
   307   which may not hold 
   308 \<close>
   308 \<close>
   309 lemma err_semilat_UnionI:
   309 lemma err_semilat_UnionI:
   310   "\<lbrakk> \<forall>A\<in>AS. err_semilat(A, r, f); AS \<noteq> {}; 
   310   "\<lbrakk> \<forall>A\<in>AS. err_semilat(A, r, f); AS \<noteq> {}; 
   311       \<forall>A\<in>AS. \<forall>B\<in>AS. A\<noteq>B \<longrightarrow> (\<forall>a\<in>A. \<forall>b\<in>B. \<not> a <=_r b & a +_f b = Err) \<rbrakk> 
   311       \<forall>A\<in>AS. \<forall>B\<in>AS. A\<noteq>B \<longrightarrow> (\<forall>a\<in>A. \<forall>b\<in>B. \<not> a <=_r b & a +_f b = Err) \<rbrakk>