tuned proof
authordesharna
Tue, 11 Jun 2024 10:27:35 +0200
changeset 80345 7d4cd57cd955
parent 80344 f05a71fa1a3f
child 80346 b5b2f651a263
tuned proof
src/HOL/Library/Multiset.thy
--- a/src/HOL/Library/Multiset.thy	Tue Jun 11 10:30:55 2024 +0200
+++ b/src/HOL/Library/Multiset.thy	Tue Jun 11 10:27:35 2024 +0200
@@ -3695,10 +3695,10 @@
   by simp
 
 lemma wfp_less_multiset[simp]:
-  assumes wfp_less: "wfp ((<) :: ('a :: preorder) \<Rightarrow> 'a \<Rightarrow> bool)"
+  assumes wf: "wfp ((<) :: ('a :: preorder) \<Rightarrow> 'a \<Rightarrow> bool)"
   shows "wfp ((<) :: 'a multiset \<Rightarrow> 'a multiset \<Rightarrow> bool)"
   unfolding less_multiset_def
-  using wfp_multp[OF wfp_less] .
+  using wfp_multp[OF wf] .
 
 
 subsubsection \<open>Strict total-order properties\<close>