src/HOL/Isar_examples/MutilatedCheckerboard.thy
changeset 16417 9bc16273c2d4
parent 13187 e5434b822a96
child 18153 a084aa91f701
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4                 Lawrence C Paulson, Cambridge University Computer Laboratory (original scripts)
     4                 Lawrence C Paulson, Cambridge University Computer Laboratory (original scripts)
     5 *)
     5 *)
     6 
     6 
     7 header {* The Mutilated Checker Board Problem *}
     7 header {* The Mutilated Checker Board Problem *}
     8 
     8 
     9 theory MutilatedCheckerboard = Main:
     9 theory MutilatedCheckerboard imports Main begin
    10 
    10 
    11 text {*
    11 text {*
    12  The Mutilated Checker Board Problem, formalized inductively.  See
    12  The Mutilated Checker Board Problem, formalized inductively.  See
    13  \cite{paulson-mutilated-board} and
    13  \cite{paulson-mutilated-board} and
    14  \url{http://isabelle.in.tum.de/library/HOL/Induct/Mutil.html} for the
    14  \url{http://isabelle.in.tum.de/library/HOL/Induct/Mutil.html} for the