src/HOLCF/Up.thy
changeset 25922 cb04d05e95fb
parent 25921 0ca392ab7f37
child 26027 87cb69d27558
equal deleted inserted replaced
25921:0ca392ab7f37 25922:cb04d05e95fb
   115 by (case_tac z, simp_all)
   115 by (case_tac z, simp_all)
   116 
   116 
   117 lemma up_lemma2:
   117 lemma up_lemma2:
   118   "\<lbrakk>chain Y; Y j \<noteq> Ibottom\<rbrakk> \<Longrightarrow> Y (i + j) \<noteq> Ibottom"
   118   "\<lbrakk>chain Y; Y j \<noteq> Ibottom\<rbrakk> \<Longrightarrow> Y (i + j) \<noteq> Ibottom"
   119 apply (erule contrapos_nn)
   119 apply (erule contrapos_nn)
   120 apply (drule_tac x="j" and y="i + j" in chain_mono3)
   120 apply (drule_tac i="j" and j="i + j" in chain_mono)
   121 apply (rule le_add2)
   121 apply (rule le_add2)
   122 apply (case_tac "Y j")
   122 apply (case_tac "Y j")
   123 apply assumption
   123 apply assumption
   124 apply simp
   124 apply simp
   125 done
   125 done