src/Doc/Prog_Prove/Isar.thy
changeset 58502 d37c712cc01b
parent 58486 f62a887c3ae7
child 58504 5f88c142676d
--- a/src/Doc/Prog_Prove/Isar.thy	Tue Sep 30 16:40:03 2014 +0200
+++ b/src/Doc/Prog_Prove/Isar.thy	Tue Sep 30 18:44:01 2014 +0200
@@ -546,7 +546,7 @@
 
 Sometimes one would like to prove some lemma locally within a proof,
 a lemma that shares the current context of assumptions but that
-has its own assumptions and is generalised over its locally fixed
+has its own assumptions and is generalized over its locally fixed
 variables at the end. This is what a \concept{raw proof block} does:
 \begin{quote}\index{$IMP053@@{text"{ ... }"} (proof block)}
 @{text"{"} \isacom{fix} @{text"x\<^sub>1 \<dots> x\<^sub>n"}\\
@@ -1031,7 +1031,7 @@
 \isacom{lemma} @{text[source]"I x y z \<Longrightarrow> x = r \<Longrightarrow> y = s \<Longrightarrow> z = t \<Longrightarrow> \<dots>"}
 \end{isabelle}
 Standard rule induction will work fine now, provided the free variables in
-@{text r}, @{text s}, @{text t} are generalised via @{text"arbitrary"}.
+@{text r}, @{text s}, @{text t} are generalized via @{text"arbitrary"}.
 
 However, induction can do the above transformation for us, behind the curtains, so we never
 need to see the expanded version of the lemma. This is what we need to write: