Skip to content

Commit

Permalink
Rename v to x in statement of transition_from_repeated_receive
Browse files Browse the repository at this point in the history
  • Loading branch information
javierdiaz72 committed May 24, 2022
1 parent 7a7c10b commit 2ef937d
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Thorn_Calculus-Semantics-Synchronous.thy
Expand Up @@ -197,7 +197,7 @@ lemmas [induct_simp] =
lemma transition_from_repeated_receive:
assumes "A \<triangleright>\<^sup>\<infinity> x. \<P> x \<rightarrow>\<^sub>s\<lparr>\<alpha>\<rparr> Q"
obtains n and X
where "\<alpha> = A \<triangleright> \<star>\<^bsup>n\<^esup> X" and "Q = post_receive n X (\<lambda>v. \<P> v \<parallel> A \<triangleright>\<^sup>\<infinity> x. \<P> x)"
where "\<alpha> = A \<triangleright> \<star>\<^bsup>n\<^esup> X" and "Q = post_receive n X (\<lambda>x. \<P> x \<parallel> A \<triangleright>\<^sup>\<infinity> x. \<P> x)"
using assms
by
(subst (asm) (2) repeated_receive_proper_def)
Expand Down

0 comments on commit 2ef937d

Please sign in to comment.