src/HOL/Library/FSet.thy
changeset 76281 457f1cba78fb
parent 76269 cee0b9fccf6f
child 76305 44b0b22f4e2e
--- a/src/HOL/Library/FSet.thy	Thu Oct 13 10:44:27 2022 +0200
+++ b/src/HOL/Library/FSet.thy	Thu Oct 13 14:27:15 2022 +0200
@@ -559,7 +559,7 @@
 lemma fimage_strict_mono:
   assumes "inj_on f (fset B)" and "A |\<subset>| B"
   shows "f |`| A |\<subset>| f |`| B"
-  \<comment> \<open>TODO: Configure transfer framework to lift @{thm Fun.inj_on_strict_subset}.\<close>
+  \<comment> \<open>TODO: Configure transfer framework to lift @{thm Fun.image_strict_mono}.\<close>
 proof (rule pfsubsetI)
   from \<open>A |\<subset>| B\<close> have "A |\<subseteq>| B"
     by (rule pfsubset_imp_fsubset)