tuned;
authorwenzelm
Thu, 22 Apr 1999 13:03:46 +0200
changeset 6480 c58bc3d2ba0f
parent 6479 b0448cab1b1e
child 6481 dbf2d9b3d6c8
tuned;
src/HOL/Isar_examples/ExprCompiler.thy
--- a/src/HOL/Isar_examples/ExprCompiler.thy	Thu Apr 22 13:03:10 1999 +0200
+++ b/src/HOL/Isar_examples/ExprCompiler.thy	Thu Apr 22 13:03:46 1999 +0200
@@ -105,13 +105,13 @@
 
 lemma exec_append:
   "ALL stack. exec (xs @ ys) stack env = exec ys (exec xs stack env) env" (is "??P xs");
-proof ("induct" ??P xs type: list);
+proof (induct ??P xs type: list);
   show "??P []"; by simp;
 
   fix x xs;
   assume "??P xs";
   show "??P (x # xs)" (is "??Q x");
-  proof ("induct" ??Q x type: instr);
+  proof (induct ??Q x type: instr);
     fix val; show "??Q (Const val)"; by brute_force;
     next;
     fix adr; show "??Q (Load adr)"; by brute_force;
@@ -123,7 +123,7 @@
 
 lemma exec_comp:
   "ALL stack. exec (comp e) stack env = eval e env # stack" (is "??P e");
-proof ("induct" ??P e type: expr);
+proof (induct ??P e type: expr);
 
   fix adr; show "??P (Variable adr)"; by brute_force;
   next;