src/ZF/IMP/Equiv.thy
changeset 46822 95f1e700b712
parent 40945 b8703f63bfb2
child 58871 c399ae4b836f
--- a/src/ZF/IMP/Equiv.thy	Tue Mar 06 16:06:52 2012 +0000
+++ b/src/ZF/IMP/Equiv.thy	Tue Mar 06 16:46:27 2012 +0000
@@ -8,7 +8,7 @@
 
 lemma aexp_iff [rule_format]:
   "[| a \<in> aexp; sigma: loc -> nat |] 
-    ==> ALL n. <a,sigma> -a-> n <-> A(a,sigma) = n"
+    ==> \<forall>n. <a,sigma> -a-> n \<longleftrightarrow> A(a,sigma) = n"
   apply (erule aexp.induct)
      apply (force intro!: evala.intros)+
   done
@@ -27,7 +27,7 @@
 
 lemma bexp_iff [rule_format]:
   "[| b \<in> bexp; sigma: loc -> nat |] 
-    ==> ALL w. <b,sigma> -b-> w <-> B(b,sigma) = w"
+    ==> \<forall>w. <b,sigma> -b-> w \<longleftrightarrow> B(b,sigma) = w"
   apply (erule bexp.induct) 
   apply (auto intro!: evalb.intros)
   done