src/Doc/Implementation/ML.thy
changeset 56594 e3a06699a13f
parent 56579 4c94f631c595
child 57347 5c8f4a35d8d7
--- a/src/Doc/Implementation/ML.thy	Tue Apr 15 19:51:55 2014 +0200
+++ b/src/Doc/Implementation/ML.thy	Tue Apr 15 20:24:49 2014 +0200
@@ -758,7 +758,7 @@
   the redundant tuple structure needs to be accommodated by formal
   reasoning.}
 
-  Currying gives some flexiblity due to \emph{partial application}.  A
+  Currying gives some flexibility due to \emph{partial application}.  A
   function @{text "f: \<tau>\<^sub>1 \<rightarrow> \<tau>\<^sub>2 \<rightarrow> \<tau>"} can be applied to @{text "x: \<tau>\<^sub>1"}
   and the remaining @{text "(f x): \<tau>\<^sub>2 \<rightarrow> \<tau>"} passed to another function
   etc.  How well this works in practice depends on the order of