typo
authornipkow
Thu, 13 Sep 2018 06:36:00 +0200
changeset 68983 caedabd2771c
parent 68980 5717fbc55521
child 68984 b1d106c1edac
typo
src/HOL/Library/Multiset.thy
--- a/src/HOL/Library/Multiset.thy	Wed Sep 12 18:44:31 2018 +0200
+++ b/src/HOL/Library/Multiset.thy	Thu Sep 13 06:36:00 2018 +0200
@@ -2652,7 +2652,7 @@
     @ sort [x\<leftarrow>xs. x > xs ! (length xs div 2)]" (is "sort ?lhs = ?rhs")
   using sort_key_by_quicksort [of "\<lambda>x. x", symmetric] by simp
 
-text \<open>A stable parametrized quicksort\<close>
+text \<open>A stable parameterized quicksort\<close>
 
 definition part :: "('b \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'b list \<Rightarrow> 'b list \<times> 'b list \<times> 'b list" where
   "part f pivot xs = ([x \<leftarrow> xs. f x < pivot], [x \<leftarrow> xs. f x = pivot], [x \<leftarrow> xs. pivot < f x])"