diff -r ef1e0cb80fde -r 949d93804740 src/Doc/Main/Main_Doc.thy --- a/src/Doc/Main/Main_Doc.thy Tue May 22 14:12:15 2018 +0200 +++ b/src/Doc/Main/Main_Doc.thy Tue May 22 11:08:37 2018 +0200 @@ -572,7 +572,6 @@ @{term"[m..[e. x \ xs]\ & @{term"map (%x. e) xs"}\\ -@{term"[x \ xs. b]"} & @{term[source]"filter (\x. b) xs"} \\ @{term"xs[n := x]"} & @{term[source]"list_update xs n x"}\\ @{term"\x\xs. e"} & @{term[source]"listsum (map (\x. e) xs)"}\\ \end{supertabular}