diff -r 0ce594837524 -r fa53d267dab3 src/HOL/Isar_Examples/Puzzle.thy --- a/src/HOL/Isar_Examples/Puzzle.thy Thu Jul 01 14:32:57 2010 +0200 +++ b/src/HOL/Isar_Examples/Puzzle.thy Thu Jul 01 18:31:46 2010 +0200 @@ -4,17 +4,13 @@ imports Main begin -text_raw {* - \footnote{A question from ``Bundeswettbewerb Mathematik''. Original - pen-and-paper proof due to Herbert Ehler; Isabelle tactic script by - Tobias Nipkow.} -*} +text_raw {* \footnote{A question from ``Bundeswettbewerb Mathematik''. + Original pen-and-paper proof due to Herbert Ehler; Isabelle tactic + script by Tobias Nipkow.} *} -text {* - \textbf{Problem.} Given some function $f\colon \Nat \to \Nat$ such - that $f \ap (f \ap n) < f \ap (\idt{Suc} \ap n)$ for all $n$. - Demonstrate that $f$ is the identity. -*} +text {* \textbf{Problem.} Given some function $f\colon \Nat \to \Nat$ + such that $f \ap (f \ap n) < f \ap (\idt{Suc} \ap n)$ for all $n$. + Demonstrate that $f$ is the identity. *} theorem assumes f_ax: "\n. f (f n) < f (Suc n)"