src/HOL/Library/Multiset.thy
changeset 74868 2741ef11ccf6
parent 74865 b5031a8f7718
child 75457 cbf011677235
--- a/src/HOL/Library/Multiset.thy	Sun Nov 28 09:57:48 2021 +0100
+++ b/src/HOL/Library/Multiset.thy	Sun Nov 28 19:12:48 2021 +0100
@@ -3193,6 +3193,12 @@
   shows "M < M \<Longrightarrow> R"
   by simp
 
+lemma wfP_less_multiset[simp]:
+  assumes wfP_less: "wfP ((<) :: ('a :: preorder) \<Rightarrow> 'a \<Rightarrow> bool)"
+  shows "wfP ((<) :: 'a multiset \<Rightarrow> 'a multiset \<Rightarrow> bool)"
+  using wfP_multp[OF wfP_less] less_multiset_def
+  by (metis wfPUNIVI wfP_induct)
+
 
 subsection \<open>Quasi-executable version of the multiset extension\<close>