Skip to content

Commit

Permalink
minor edits
Browse files Browse the repository at this point in the history
  • Loading branch information
Andrei Popescu committed Oct 15, 2024
1 parent 9550727 commit 3328d50
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion thys/POPLmark/SystemFSub.thy
Original file line number Diff line number Diff line change
Expand Up @@ -78,7 +78,7 @@ corollary Forall_inject_same[simp]: "Forall X T1 T2 = Forall X S1 S2 \<longleftr

lemma Forall_rrename:
assumes "bij \<sigma>" "|supp \<sigma>| <o |UNIV::'a set|" shows "
(\<And>a'. a'\<in>FFVars_typ T2 - {x::'a::var_typ_pre} \<Longrightarrow> \<sigma> a' = a') \<Longrightarrow> Forall x T1 T2 = Forall (\<sigma> x) T1 (rrename_typ \<sigma> T2)"
(\<And>Y. Y\<in>FFVars_typ T2 - {X::'a::var_typ_pre} \<Longrightarrow> \<sigma> Y = Y) \<Longrightarrow> Forall X T1 T2 = Forall (\<sigma> X) T1 (rrename_typ \<sigma> T2)"
apply (unfold Forall_def)
apply (unfold typ.TT_injects0)
apply (unfold set3_typ_pre_def set2_typ_pre_def comp_def Abs_typ_pre_inverse[OF UNIV_I] map_sum.simps
Expand Down

0 comments on commit 3328d50

Please sign in to comment.