added lemma
authornipkow
Thu, 20 Jun 2013 17:43:36 +0200
changeset 52401 56e83c57f953
parent 52400 ded7b9c60dc2
child 52402 c2f30ba4bb98
added lemma
src/HOL/IMP/Denotational.thy
--- a/src/HOL/IMP/Denotational.thy	Thu Jun 20 17:26:16 2013 +0200
+++ b/src/HOL/IMP/Denotational.thy	Thu Jun 20 17:43:36 2013 +0200
@@ -59,6 +59,9 @@
   "(s,t) \<in> D(c)  =  ((c,s) \<Rightarrow> t)"
 by (metis D_if_big_step Big_step_if_D[simplified])
 
+corollary equiv_c_iff_equal_D: "(c1 \<sim> c2) \<longleftrightarrow> D c1 = D c2"
+by(simp add: denotational_is_big_step[symmetric] set_eq_iff)
+
 
 subsection "Continuity"