src/Doc/Prog_Prove/Logic.thy
changeset 58502 d37c712cc01b
parent 56989 fafcf43ded4a
child 58504 5f88c142676d
--- a/src/Doc/Prog_Prove/Logic.thy	Tue Sep 30 16:40:03 2014 +0200
+++ b/src/Doc/Prog_Prove/Logic.thy	Tue Sep 30 18:44:01 2014 +0200
@@ -793,7 +793,7 @@
 \subsection*{Exercises}
 
 \begin{exercise}
-Formalise the following definition of palindromes
+Formalize the following definition of palindromes
 \begin{itemize}
 \item The empty list and a singleton list are palindromes.
 \item If @{text xs} is a palindrome, so is @{term "a # xs @ [a]"}.