diff -r ceb0bdc99893 -r 6c722e960f2e thys/Hoare_gen.thy --- a/thys/Hoare_gen.thy Fri Mar 21 21:40:51 2014 +0800 +++ b/thys/Hoare_gen.thy Fri Mar 21 13:49:20 2014 +0000 @@ -12,7 +12,7 @@ where "pasrt b = (\ s . s = 0 \ b)" -(* smae as sep.mult.left_commute *) +(* same as sep.mult.left_commute *) lemma sep_conj_cond1: "(p \* \* q) = ( \* p \* q)" by (rule sep.mult.left_commute) @@ -289,15 +289,15 @@ by (smt IHoare_def code_exI) lemma I_code_extension: - assumes h: "I. \ P \ c \ Q \" - shows "I. \ P \ c ** e \ Q \" + assumes h: "I. \P\ c \Q\" + shows "I. \P\ c \* e \Q\" using h by (smt IHoare_def sep_exec.code_extension) lemma I_composition: assumes h1: "I. \P\ c1 \Q\" and h2: "I. \Q\ c2 \R\" - shows "I. \P\ c1 ** c2 \R\" + shows "I. \P\ c1 \* c2 \R\" using h1 h2 by (smt IHoare_def sep_exec.composition)