src/HOL/Hoare/Hoare_Logic.thy
changeset 38353 d98baa2cf589
parent 37591 d3daea901123
child 41959 b460124855b8
--- a/src/HOL/Hoare/Hoare_Logic.thy	Wed Aug 11 18:22:14 2010 +0200
+++ b/src/HOL/Hoare/Hoare_Logic.thy	Wed Aug 11 18:41:06 2010 +0200
@@ -41,8 +41,8 @@
   "Sem (Basic f) s s'" "Sem (c1;c2) s s'"
   "Sem (IF b THEN c1 ELSE c2 FI) s s'"
 
-definition Valid :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a bexp \<Rightarrow> bool" where
-  "Valid p c q == !s s'. Sem c s s' --> s : p --> s' : q"
+definition Valid :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a bexp \<Rightarrow> bool"
+  where "Valid p c q \<longleftrightarrow> (!s s'. Sem c s s' --> s : p --> s' : q)"