src/HOL/IMP/Hoare_Examples.thy
changeset 47818 151d137f1095
parent 45015 fdac1e9880eb
child 50986 c54ea7f5418f
--- a/src/HOL/IMP/Hoare_Examples.thy	Fri Apr 27 23:17:58 2012 +0200
+++ b/src/HOL/IMP/Hoare_Examples.thy	Sat Apr 28 07:38:22 2012 +0200
@@ -51,17 +51,17 @@
 pulling back the postcondition towards the precondition. *}
 
 lemma "\<turnstile> {\<lambda>s. 0 <= n} ''x'' ::= N 0; ''y'' ::= N 0; w n {\<lambda>s. s ''x'' = \<Sum> {1 .. n}}"
-apply(rule hoare.Semi)
+apply(rule hoare.Seq)
 prefer 2
 apply(rule While'
   [where P = "\<lambda>s. s ''x'' = \<Sum> {1..s ''y''} \<and> 0 \<le> s ''y'' \<and> s ''y'' \<le> n"])
-apply(rule Semi)
+apply(rule Seq)
 prefer 2
 apply(rule Assign)
 apply(rule Assign')
 apply(fastforce simp: atLeastAtMostPlus1_int_conv algebra_simps)
 apply(fastforce)
-apply(rule Semi)
+apply(rule Seq)
 prefer 2
 apply(rule Assign)
 apply(rule Assign')