src/Doc/Prog_Prove/Bool_nat_list.thy
changeset 59360 b1e5d552e8cc
parent 59204 0cbe0a56d3fa
child 62222 54a7b9422d3e
--- a/src/Doc/Prog_Prove/Bool_nat_list.thy	Wed Jan 14 15:22:50 2015 +0100
+++ b/src/Doc/Prog_Prove/Bool_nat_list.thy	Wed Jan 14 17:04:19 2015 +0100
@@ -397,7 +397,7 @@
 @{text"length :: 'a list \<Rightarrow> nat"}\index{length@@{const length}} (with the obvious definition),
 and the \indexed{@{const map}}{map} function that applies a function to all elements of a list:
 \begin{isabelle}
-\isacom{fun} @{const map} @{text"::"} @{typ[source] "('a \<Rightarrow> 'b) \<Rightarrow> 'a list \<Rightarrow> 'b list"}\\
+\isacom{fun} @{const map} @{text"::"} @{typ[source] "('a \<Rightarrow> 'b) \<Rightarrow> 'a list \<Rightarrow> 'b list"} \isacom{where}\\
 @{text"\""}@{thm list.map(1) [of f]}@{text"\" |"}\\
 @{text"\""}@{thm list.map(2) [of f x xs]}@{text"\""}
 \end{isabelle}