src/HOL/MicroJava/BV/SemilatAlg.thy
changeset 23281 e26ec695c9b3
parent 16417 9bc16273c2d4
child 23464 bc2563c37b1a
--- a/src/HOL/MicroJava/BV/SemilatAlg.thy	Wed Jun 06 19:12:40 2007 +0200
+++ b/src/HOL/MicroJava/BV/SemilatAlg.thy	Wed Jun 06 19:12:59 2007 +0200
@@ -156,7 +156,7 @@
 
 lemma ub1': includes semilat
 shows "\<lbrakk>\<forall>(p,s) \<in> set S. s \<in> A; y \<in> A; (a,b) \<in> set S\<rbrakk> 
-  \<Longrightarrow> b <=_r map snd [(p', t')\<in>S. p' = a] ++_f y" 
+  \<Longrightarrow> b <=_r map snd [(p', t')\<leftarrow>S. p' = a] ++_f y" 
 proof -
   let "b <=_r ?map ++_f y" = ?thesis
 
@@ -175,7 +175,7 @@
 
 lemma plusplus_empty:  
   "\<forall>s'. (q, s') \<in> set S \<longrightarrow> s' +_f ss ! q = ss ! q \<Longrightarrow>
-   (map snd [(p', t')\<in> S. p' = q] ++_f ss ! q) = ss ! q"
+   (map snd [(p', t') \<leftarrow> S. p' = q] ++_f ss ! q) = ss ! q"
 apply (induct S)
 apply auto 
 done