diff -r 28df61d931e2 -r a455e69c31cc src/HOL/Induct/Mutil.thy --- a/src/HOL/Induct/Mutil.thy Wed Jul 11 11:13:08 2007 +0200 +++ b/src/HOL/Induct/Mutil.thy Wed Jul 11 11:14:51 2007 +0200 @@ -15,18 +15,19 @@ the Mutilated Checkerboard Problem by J McCarthy. *} -consts tiling :: "'a set set => 'a set set" -inductive "tiling A" - intros +inductive_set + tiling :: "'a set set => 'a set set" + for A :: "'a set set" + where empty [simp, intro]: "{} \ tiling A" - Un [simp, intro]: "[| a \ A; t \ tiling A; a \ t = {} |] + | Un [simp, intro]: "[| a \ A; t \ tiling A; a \ t = {} |] ==> a \ t \ tiling A" -consts domino :: "(nat \ nat) set set" -inductive domino - intros +inductive_set + domino :: "(nat \ nat) set set" + where horiz [simp]: "{(i, j), (i, Suc j)} \ domino" - vertl [simp]: "{(i, j), (Suc i, j)} \ domino" + | vertl [simp]: "{(i, j), (Suc i, j)} \ domino" text {* \medskip Sets of squares of the given colour*}