src/Doc/Main/Main_Doc.thy
changeset 68249 949d93804740
parent 68224 1f7308050349
child 68364 5c579bb9adb1
--- 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..<n]"} & @{term[source]"upt m n"}\\
 @{term"[i..j]"} & @{term[source]"upto i j"}\\
 \<open>[e. x \<leftarrow> xs]\<close> & @{term"map (%x. e) xs"}\\
-@{term"[x \<leftarrow> xs. b]"} & @{term[source]"filter (\<lambda>x. b) xs"} \\
 @{term"xs[n := x]"} & @{term[source]"list_update xs n x"}\\
 @{term"\<Sum>x\<leftarrow>xs. e"} & @{term[source]"listsum (map (\<lambda>x. e) xs)"}\\
 \end{supertabular}