src/HOL/Library/Poly_Mapping.thy
changeset 76484 defaa0b17424
parent 75455 91c16c5ad3e9
child 76987 4c275405faae
--- a/src/HOL/Library/Poly_Mapping.thy	Sun Nov 06 23:10:28 2022 +0100
+++ b/src/HOL/Library/Poly_Mapping.thy	Mon Nov 07 22:16:37 2022 +0100
@@ -1487,7 +1487,7 @@
   shows "items (the_value xs) = xs"
 proof -
   from assms have "sorted_list_of_set (set (List.map fst xs)) = List.map fst xs"
-    unfolding sorted_list_of_set_sort_remdups by (simp add: distinct_remdups_id sorted_sort_id)
+    unfolding sorted_list_of_set_sort_remdups by (simp add: distinct_remdups_id sort_key_id_if_sorted)
   moreover from assms have "keys (the_value xs) = fst ` set xs"
     by transfer (auto simp add: image_def split: option.split dest: set_map_of_compr)
   ultimately show ?thesis