equal
deleted
inserted
replaced
1 (* Title: HOL/Isar_examples/MutilatedCheckerboard.thy |
1 (* Title: HOL/Isar_examples/MutilatedCheckerboard.thy |
2 ID: $Id$ |
2 ID: $Id$ |
3 Author: Markus Wenzel, TU Muenchen (Isar document) |
3 Author: Markus Wenzel, TU Muenchen (Isar document) |
4 Lawrence C Paulson, Cambridge University Computer Laboratory (original scripts) |
4 Lawrence C Paulson, Cambridge University Computer Laboratory (original scripts) |
5 |
|
6 The Mutilated Checker Board Problem, formalized inductively. |
|
7 Originator is Max Black, according to J A Robinson. |
|
8 Popularized as the Mutilated Checkerboard Problem by J McCarthy. |
|
9 |
|
10 See also HOL/Induct/Mutil for the original Isabelle tactic scripts. |
|
11 *) |
5 *) |
12 |
6 |
13 header {* The Mutilated Checker Board Problem *}; |
7 header {* The Mutilated Checker Board Problem *}; |
14 |
8 |
15 theory MutilatedCheckerboard = Main:; |
9 theory MutilatedCheckerboard = Main:; |
16 |
10 |
|
11 text {* |
|
12 The Mutilated Checker Board Problem, formalized inductively. See |
|
13 \cite{paulson-mutilated-board} and |
|
14 \url{http://isabelle.in.tum.de/library/HOL/Induct/Mutil.html} for the |
|
15 original tactic script version. |
|
16 *}; |
17 |
17 |
18 subsection {* Tilings *}; |
18 subsection {* Tilings *}; |
19 |
19 |
20 consts |
20 consts |
21 tiling :: "'a set set => 'a set set"; |
21 tiling :: "'a set set => 'a set set"; |