Skip to content

Commit

Permalink
rename variables for rsubst2 squash
Browse files Browse the repository at this point in the history
Signed-off-by: Michael McInerney <[email protected]>
  • Loading branch information
michaelmcinerney committed Apr 8, 2024
1 parent 01c6bd0 commit 455faf5
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion lib/Lib.thy
Original file line number Diff line number Diff line change
Expand Up @@ -2536,7 +2536,7 @@ qed
lemmas rsubst = back_subst[where a=s and b=t for s t]

lemma rsubst2:
"\<lbrakk>P s x; s = t; x = y\<rbrakk> \<Longrightarrow> P t y"
"\<lbrakk>P a b; a = s; b = t\<rbrakk> \<Longrightarrow> P s t"
by simp

lemma rsubst3:
Expand Down

0 comments on commit 455faf5

Please sign in to comment.