src/HOL/UNITY/Comp/Priority.thy
changeset 69597 ff784d5a5bfb
parent 67613 ce654b0e6d69
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   252 apply (blast intro: above_decreases_psp')+
   252 apply (blast intro: above_decreases_psp')+
   253 done
   253 done
   254 
   254 
   255 
   255 
   256 text\<open>We have proved all (relevant) theorems given in the paper.  We didn't
   256 text\<open>We have proved all (relevant) theorems given in the paper.  We didn't
   257 assume any thing about the relation @{term r}.  It is not necessary that
   257 assume any thing about the relation \<^term>\<open>r\<close>.  It is not necessary that
   258 @{term r} be a priority relation as assumed in the original proof.  It
   258 \<^term>\<open>r\<close> be a priority relation as assumed in the original proof.  It
   259 suffices that we start from a state which is finite and acyclic.\<close>
   259 suffices that we start from a state which is finite and acyclic.\<close>
   260 
   260 
   261 
   261 
   262 end
   262 end