Skip to content

Commit

Permalink
remove extra space and rename variable in corres_cross_add_guard
Browse files Browse the repository at this point in the history
Signed-off-by: Michael McInerney <[email protected]>
  • Loading branch information
michaelmcinerney committed Mar 27, 2024
1 parent d593972 commit a53b39b
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions lib/Corres_UL.thy
Original file line number Diff line number Diff line change
Expand Up @@ -1177,8 +1177,8 @@ lemma corres_move_asm:
lemmas corres_cross_over_guard = corres_move_asm[rotated]

lemma corres_cross_add_guard:
"\<lbrakk> \<And>s s'. \<lbrakk>(s,s') \<in> sr; P s; P' s'\<rbrakk> \<Longrightarrow> Q s';
corres_underlying sr nf nf' r P (P' and Q) f g\<rbrakk>
"\<lbrakk> \<And>s s'. \<lbrakk>(s,s') \<in> sr; P s; P' s'\<rbrakk> \<Longrightarrow> Q' s';
corres_underlying sr nf nf' r P (P' and Q') f g\<rbrakk>
\<Longrightarrow> corres_underlying sr nf nf' r P P' f g"
by (fastforce simp: corres_underlying_def)

Expand Down

0 comments on commit a53b39b

Please sign in to comment.