changeset 81113 | 6fefd6c602fa |
parent 73477 | 1d8a79aa2a99 |
--- a/src/HOL/Library/Disjoint_FSets.thy Fri Oct 04 13:22:35 2024 +0200 +++ b/src/HOL/Library/Disjoint_FSets.thy Fri Oct 04 13:29:33 2024 +0200 @@ -62,7 +62,7 @@ (* FIXME should be provable without lifting *) lemma fmadd_disjnt: "fdisjnt (fmdom m) (fmdom n) \<Longrightarrow> m ++\<^sub>f n = n ++\<^sub>f m" unfolding fdisjnt_alt_def -including fset.lifting fmap.lifting +including fset.lifting and fmap.lifting apply transfer apply (rule ext) apply (auto simp: map_add_def split: option.splits)