src/HOL/ex/Puzzle.thy
author paulson
Mon, 05 Mar 2001 15:25:11 +0100
changeset 11193 851c90b23a9e
parent 8018 bedd0beabbae
child 13116 baabb0fd2ccf
permissions -rw-r--r--
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp

(*  Title:      HOL/ex/Puzzle.thy
    ID:         $Id$
    Author:     Tobias Nipkow
    Copyright   1993 TU Muenchen

A question from "Bundeswettbewerb Mathematik"
*)

Puzzle = Main +
consts f :: nat => nat
rules  f_ax "f(f(n)) < f(Suc(n))"
end