src/HOL/Isar_examples/MutilatedCheckerboard.thy
changeset 7968 964b65b4e433
parent 7874 180364256231
child 8281 188e2924433e
equal deleted inserted replaced
7967:942274e0f7a8 7968:964b65b4e433
     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";