src/HOL/Bali/DefiniteAssignmentCorrect.thy
changeset 18459 2b102759160d
parent 18447 da548623916a
child 18576 8d98b7711e47
--- a/src/HOL/Bali/DefiniteAssignmentCorrect.thy	Thu Dec 22 00:28:39 2005 +0100
+++ b/src/HOL/Bali/DefiniteAssignmentCorrect.thy	Thu Dec 22 00:28:41 2005 +0100
@@ -105,7 +105,7 @@
     have True and True and 
        "\<And> jmps' jmps. \<lbrakk>jumpNestingOkS jmps' c; jmps' \<subseteq> jmps\<rbrakk> \<Longrightarrow> jumpNestingOkS jmps c" 
        and True
-  proof (induct rule: var_expr_stmt.induct)
+  proof (induct rule: var_expr_stmt.inducts)
     case (Lab j c jmps' jmps)
     have jmpOk: "jumpNestingOkS jmps' (j\<bullet> c)" .
     have jmps: "jmps' \<subseteq> jmps" .
@@ -2017,7 +2017,7 @@
         "\<And> c v s0 s. \<lbrakk> constVal e = Some c; G\<turnstile>Norm s0 \<midarrow>e-\<succ>v\<rightarrow> s\<rbrakk> 
                       \<Longrightarrow> v = c \<and> normal s"
         and True and True
-  proof (induct  rule: var_expr_stmt.induct)
+  proof (induct  rule: var_expr_stmt.inducts)
     case NewC hence False by simp thus ?case ..
   next
     case NewA hence False by simp thus ?case ..
@@ -2165,7 +2165,7 @@
        "\<And> c. \<lbrakk>constVal e = Some c;Env\<turnstile>e\<Colon>-PrimT Boolean\<rbrakk> 
                 \<Longrightarrow> typeof empty_dt c = Some (PrimT Boolean)"
        and True and True 
-  proof (induct rule: var_expr_stmt.induct)
+  proof (induct rule: var_expr_stmt.inducts)
     case NewC hence False by simp thus ?case ..
   next
     case NewA hence False by simp thus ?case ..