diff -r b35ffbe82031 -r 11a24dab1880 src/HOL/List.thy --- a/src/HOL/List.thy Mon Dec 19 15:54:03 2022 +0100 +++ b/src/HOL/List.thy Mon Dec 19 16:00:49 2022 +0100 @@ -5535,7 +5535,7 @@ next assume ?R have "i < j \ j < length xs \ P (xs ! i) (xs ! j)" for i j - by(induct i j rule: less_Suc_induct)(simp add: \?R\, meson assms transpE transp_less) + by(induct i j rule: less_Suc_induct)(simp add: \?R\, meson assms transpE transp_on_less) thus ?L by (simp add: sorted_wrt_iff_nth_less) qed