src/HOL/Library/Finite_Map.thy
changeset 69700 7a92cbec7030
parent 69593 3dda49e08b9d
child 70277 ac24aaf84a36
--- a/src/HOL/Library/Finite_Map.thy	Sun Jan 20 17:15:49 2019 +0000
+++ b/src/HOL/Library/Finite_Map.thy	Mon Jan 21 14:44:23 2019 +0000
@@ -1406,7 +1406,7 @@
   moreover have "inj (inv fmap_of_list)"
     using fmap_of_list_surj by (rule surj_imp_inj_inv)
   ultimately have "inj (to_nat \<circ> inv fmap_of_list)"
-    by (rule inj_comp)
+    by (rule inj_compose)
   thus "\<exists>to_nat::('a, 'b) fmap \<Rightarrow> nat. inj to_nat"
     by auto
 qed