src/HOL/Isar_examples/MutilatedCheckerboard.thy
changeset 8281 188e2924433e
parent 7968 964b65b4e433
child 8297 f5fdb69ad4d2
--- a/src/HOL/Isar_examples/MutilatedCheckerboard.thy	Tue Feb 22 21:49:34 2000 +0100
+++ b/src/HOL/Isar_examples/MutilatedCheckerboard.thy	Tue Feb 22 21:50:02 2000 +0100
@@ -35,7 +35,7 @@
 proof;
   assume "t : tiling A" (is "_ : ?T");
   thus "u : ?T --> t Int u = {} --> t Un u : ?T" (is "?P t");
-  proof (induct t set: tiling);
+  proof (induct t in set: tiling);
     show "?P {}"; by simp;
 
     fix a t;
@@ -168,7 +168,7 @@
   assume b: "b < 2";
   assume "d : domino";
   thus ?thesis (is "?P d");
-  proof (induct d set: domino);
+  proof (induct d in set: domino);
     from b; have b_cases: "b = 0 | b = 1"; by arith;
     fix i j;
     note [simp] = evnodd_empty evnodd_insert mod_Suc;
@@ -192,7 +192,7 @@
 proof -;
   assume "t : ?T";
   thus "?F t";
-  proof (induct t set: tiling);
+  proof (induct t in set: tiling);
     show "?F {}"; by (rule Finites.emptyI);
     fix a t; assume "?F t";
     assume "a : domino"; hence "?F a"; by (rule domino_finite);
@@ -206,7 +206,7 @@
 proof -;
   assume "t : ?T";
   thus "?P t";
-  proof (induct t set: tiling);
+  proof (induct t in set: tiling);
     show "?P {}"; by (simp add: evnodd_def);
 
     fix a t;