src/HOL/IMP/Hoare_Sound_Complete.thy
changeset 54809 319358e48bb1
parent 53015 a1119cf551e8
child 63538 d7b5e2a222c2
--- a/src/HOL/IMP/Hoare_Sound_Complete.thy	Wed Dec 18 16:50:14 2013 +0100
+++ b/src/HOL/IMP/Hoare_Sound_Complete.thy	Wed Dec 18 17:52:44 2013 +0100
@@ -77,4 +77,7 @@
   show "\<turnstile> {wp c Q} c {Q}" by(rule wp_is_pre)
 qed
 
+corollary hoare_sound_complete: "\<turnstile> {P}c{Q} \<longleftrightarrow> \<Turnstile> {P}c{Q}"
+by (metis hoare_complete hoare_sound)
+
 end