src/HOL/IMP/Sem_Equiv.thy
changeset 52046 bc01725d7918
parent 52021 59963cda805a
child 52121 5b889b1b465b
--- a/src/HOL/IMP/Sem_Equiv.thy	Fri May 17 02:57:00 2013 +0200
+++ b/src/HOL/IMP/Sem_Equiv.thy	Fri May 17 08:19:52 2013 +0200
@@ -70,7 +70,7 @@
 lemma equiv_up_to_seq:
   "P \<Turnstile> c \<sim> c' \<Longrightarrow> Q \<Turnstile> d \<sim> d' \<Longrightarrow>
   (\<And>s s'. (c,s) \<Rightarrow> s' \<Longrightarrow> P s \<Longrightarrow> Q s') \<Longrightarrow>
-  P \<Turnstile> (c; d) \<sim> (c'; d')"
+  P \<Turnstile> (c;; d) \<sim> (c';; d')"
   by (clarsimp simp: equiv_up_to_def) blast
 
 lemma equiv_up_to_while_lemma: