# HG changeset patch # User nipkow # Date 1749901675 -7200 # Node ID 4db3f6e6fb6c4fa57fdee090e6b532ff619b0cbf # Parent e0fb460181876c6ec97afcff7a3312d277d53d64 removed pointless leftovers diff -r e0fb46018187 -r 4db3f6e6fb6c src/HOL/ex/Perm_Fragments.thy --- a/src/HOL/ex/Perm_Fragments.thy Sat Jun 14 11:45:56 2025 +0200 +++ b/src/HOL/ex/Perm_Fragments.thy Sat Jun 14 13:47:55 2025 +0200 @@ -261,36 +261,4 @@ end - -text \Misc\ - -lemma (in comm_monoid_list_set) sorted_list_of_set: - assumes "finite A" - shows "list.F (map h (sorted_list_of_set A)) = set.F h A" -proof - - from distinct_sorted_list_of_set - have "set.F h (set (sorted_list_of_set A)) = list.F (map h (sorted_list_of_set A))" - by (rule distinct_set_conv_list) - with \finite A\ show ?thesis - by (simp) -qed - -primrec subtract :: "'a list \ 'a list \ 'a list" -where - "subtract [] ys = ys" -| "subtract (x # xs) ys = subtract xs (removeAll x ys)" - -lemma length_subtract_less_eq [simp]: - "length (subtract xs ys) \ length ys" -proof (induct xs arbitrary: ys) - case Nil then show ?case by simp -next - case (Cons x xs) - then have "length (subtract xs (removeAll x ys)) \ length (removeAll x ys)" . - also have "length (removeAll x ys) \ length ys" - by simp - finally show ?case - by simp -qed - end