CpsG.thy
changeset 62 031d2ae9c9b8
parent 61 f8194fd6214f
child 63 b620a2a0806a
--- a/CpsG.thy	Fri Dec 18 22:47:32 2015 +0800
+++ b/CpsG.thy	Tue Dec 22 23:13:31 2015 +0800
@@ -10,6 +10,10 @@
        difference is the order of arguemts. *}
 definition "the_preced s th = preced th s"
 
+lemma inj_the_preced: 
+  "inj_on (the_preced s) (threads s)"
+  by (metis inj_onI preced_unique the_preced_def)
+
 text {* @{term "the_thread"} extracts thread out of RAG node. *}
 fun the_thread :: "node \<Rightarrow> thread" where
    "the_thread (Th th) = th"