src/HOL/Isar_examples/MutilatedCheckerboard.thy
changeset 7968 964b65b4e433
parent 7874 180364256231
child 8281 188e2924433e
--- a/src/HOL/Isar_examples/MutilatedCheckerboard.thy	Thu Oct 28 19:53:24 1999 +0200
+++ b/src/HOL/Isar_examples/MutilatedCheckerboard.thy	Thu Oct 28 19:57:34 1999 +0200
@@ -2,18 +2,18 @@
     ID:         $Id$
     Author:     Markus Wenzel, TU Muenchen (Isar document)
                 Lawrence C Paulson, Cambridge University Computer Laboratory (original scripts)
-
-The Mutilated Checker Board Problem, formalized inductively.
-  Originator is Max Black, according to J A Robinson.
-  Popularized as the Mutilated Checkerboard Problem by J McCarthy.
-
-See also HOL/Induct/Mutil for the original Isabelle tactic scripts.
 *)
 
 header {* The Mutilated Checker Board Problem *};
 
 theory MutilatedCheckerboard = Main:;
 
+text {*
+ The Mutilated Checker Board Problem, formalized inductively.  See
+ \cite{paulson-mutilated-board} and
+ \url{http://isabelle.in.tum.de/library/HOL/Induct/Mutil.html} for the
+ original tactic script version.
+*};
 
 subsection {* Tilings *};