diff -r 59b937edcff8 -r 4ec8e654112f src/HOL/IMP/Collecting_Examples.thy --- a/src/HOL/IMP/Collecting_Examples.thy Thu Jun 26 17:30:33 2025 +0200 +++ b/src/HOL/IMP/Collecting_Examples.thy Thu Jun 26 17:25:29 2025 +0200 @@ -7,9 +7,9 @@ subsubsection "Pretty printing state sets" text\Tweak code generation to work with sets of non-equality types:\ -declare insert_code[code del] union_coset_filter[code del] -lemma insert_code [code]: "insert x (set xs) = set (x#xs)" -by simp +lemma insert_code [code]: "insert x (set xs) = set (x#xs)" + and union_code [code]: "set xs \ A = fold insert xs A" + by (simp_all add: union_set_fold) text\Compensate for the fact that sets may now have duplicates:\ definition compact :: "'a set \ 'a set" where