diff -r 98bfff1d159d -r a6e0696d7110 src/HOL/Library/More_List.thy --- a/src/HOL/Library/More_List.thy Thu May 20 17:29:43 2010 +0200 +++ b/src/HOL/Library/More_List.thy Thu May 20 17:35:02 2010 +0200 @@ -237,7 +237,7 @@ "SUPR (set xs) f = fold (sup \ f) xs bot" unfolding SUPR_def set_map [symmetric] Sup_set_fold fold_map .. -text {* nth_map *} +text {* @{text nth_map} *} definition nth_map :: "nat \ ('a \ 'a) \ 'a list \ 'a list" where "nth_map n f xs = (if n < length xs then