PrioG.thy~
changeset 62 031d2ae9c9b8
parent 61 f8194fd6214f
child 63 b620a2a0806a
--- a/PrioG.thy~	Fri Dec 18 22:47:32 2015 +0800
+++ b/PrioG.thy~	Tue Dec 22 23:13:31 2015 +0800
@@ -2914,4 +2914,15 @@
   from the concise and miniature model of PIP given in PrioGDef.thy.
 *}
 
+lemma eq_dependants: "dependants (wq s) = dependants s"
+  by (simp add: s_dependants_abv wq_def)
+
+lemma next_th_unique: 
+  assumes nt1: "next_th s th cs th1"
+  and nt2: "next_th s th cs th2"
+  shows "th1 = th2"
+using assms by (unfold next_th_def, auto)
+
+
+ 
 end