Skip to content

Commit

Permalink
Readd syntax and size setup for labeled fset
Browse files Browse the repository at this point in the history
  • Loading branch information
jvanbruegge committed Mar 9, 2024
1 parent 08537c6 commit d532ac1
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions thys/POPLmark/Labeled_FSet.thy
Original file line number Diff line number Diff line change
Expand Up @@ -215,7 +215,7 @@ snd o MRBNF_Def.register_mrbnf_as_bnf (the (MRBNF_Def.mrbnf_of @{context} "Label
print_theorems
print_bnfs


(*
(* locale+interpretation as a trick to get automatic proofs and replace new constants
by existing ones afterwards *)
locale AUX
Expand All @@ -234,6 +234,7 @@ interpretation AUX
maps (fn f => BNF_Def.bnf_of @{context} @{type_name lfset} |> the |> f) [BNF_Def.set_defs_of_bnf,
single o BNF_Def.map_def_of_bnf, single o BNF_Def.rel_def_of_bnf])\<close>) (rule refl)+

*)
context begin

qualified definition "Rep = Rep_G o Rep_lfset"
Expand Down Expand Up @@ -360,8 +361,8 @@ lemmas size_lfset_overloaded_simps =
folded size_lfset_overloaded_def]

lemma lfset_size_o_map:
"inj f \<Longrightarrow> size_lfset (\<lambda>_. 0) g \<circ> map_lfset_id f = size_lfset (\<lambda>_. 0) (g \<circ> f)"
unfolding fun_eq_iff o_apply map_lfset_id_def
"inj f \<Longrightarrow> size_lfset (\<lambda>_. 0) g \<circ> map_lfset id f = size_lfset (\<lambda>_. 0) (g \<circ> f)"
unfolding fun_eq_iff o_apply
by transfer
(subst fun_cong[OF fset_size_o_map, unfolded o_apply],
auto simp add: inj_on_def split_beta map_prod_def size_prod_simp)
Expand Down Expand Up @@ -419,5 +420,4 @@ unfolded id_def inj_on_def, simplified, termination_simp]

hide_fact (open) FSet.bex_simps FSet.ball_simps


end

0 comments on commit d532ac1

Please sign in to comment.