src/HOL/UNITY/SubstAx.thy
changeset 61824 dcbe9f756ae0
parent 60773 d09c66a0ea10
child 61952 546958347e05
equal deleted inserted replaced
61823:5daa82ba4078 61824:dcbe9f756ae0
   359 apply (rule_tac f = f and f1 = "%k. l - k" 
   359 apply (rule_tac f = f and f1 = "%k. l - k" 
   360        in wf_less_than [THEN wf_inv_image, THEN LeadsTo_wf_induct])
   360        in wf_less_than [THEN wf_inv_image, THEN LeadsTo_wf_induct])
   361 apply (simp add: Image_singleton, clarify)
   361 apply (simp add: Image_singleton, clarify)
   362 apply (case_tac "m<l")
   362 apply (case_tac "m<l")
   363  apply (blast intro: LeadsTo_weaken_R diff_less_mono2)
   363  apply (blast intro: LeadsTo_weaken_R diff_less_mono2)
   364 apply (blast intro: not_leE subset_imp_LeadsTo)
   364 apply (blast intro: not_le_imp_less subset_imp_LeadsTo)
   365 done
   365 done
   366 
   366 
   367 
   367 
   368 subsection{*Completion: Binary and General Finite versions*}
   368 subsection{*Completion: Binary and General Finite versions*}
   369 
   369