src/HOL/IMP/Big_Step.thy
changeset 45015 fdac1e9880eb
parent 44923 b80108b346a9
child 45321 b227989b6ee6
--- a/src/HOL/IMP/Big_Step.thy	Tue Sep 20 05:47:11 2011 +0200
+++ b/src/HOL/IMP/Big_Step.thy	Tue Sep 20 05:48:23 2011 +0200
@@ -215,7 +215,7 @@
 
 text {* This proof is automatic. *}
 theorem big_step_determ: "\<lbrakk> (c,s) \<Rightarrow> t; (c,s) \<Rightarrow> u \<rbrakk> \<Longrightarrow> u = t"
-apply (induct arbitrary: u rule: big_step.induct)
+apply (induction arbitrary: u rule: big_step.induct)
 apply blast+
 done
 
@@ -225,7 +225,7 @@
 *}
 theorem
   "(c,s) \<Rightarrow> t  \<Longrightarrow>  (c,s) \<Rightarrow> t'  \<Longrightarrow>  t' = t"
-proof (induct arbitrary: t' rule: big_step.induct)
+proof (induction arbitrary: t' rule: big_step.induct)
   -- "the only interesting case, @{text WhileTrue}:"
   fix b c s s1 t t'
   -- "The assumptions of the rule:"