src/HOL/Isar_examples/MutilatedCheckerboard.thy
changeset 23746 a455e69c31cc
parent 23373 ead82c82da9e
child 26813 6a4d5ca6d2e5
--- a/src/HOL/Isar_examples/MutilatedCheckerboard.thy	Wed Jul 11 11:13:08 2007 +0200
+++ b/src/HOL/Isar_examples/MutilatedCheckerboard.thy	Wed Jul 11 11:14:51 2007 +0200
@@ -17,13 +17,12 @@
 
 subsection {* Tilings *}
 
-consts
+inductive_set
   tiling :: "'a set set => 'a set set"
-
-inductive "tiling A"
-  intros
+  for A :: "'a set set"
+  where
     empty: "{} : tiling A"
-    Un: "a : A ==> t : tiling A ==> a <= - t ==> a Un t : tiling A"
+  | Un: "a : A ==> t : tiling A ==> a <= - t ==> a Un t : tiling A"
 
 
 text "The union of two disjoint tilings is a tiling."
@@ -118,13 +117,11 @@
 
 subsection {* Dominoes *}
 
-consts
+inductive_set
   domino :: "(nat * nat) set set"
-
-inductive domino
-  intros
+  where
     horiz: "{(i, j), (i, j + 1)} : domino"
-    vertl: "{(i, j), (i + 1, j)} : domino"
+  | vertl: "{(i, j), (i + 1, j)} : domino"
 
 lemma dominoes_tile_row:
   "{i} <*> below (2 * n) : tiling domino"