src/HOL/Isar_examples/Puzzle.thy
changeset 18193 54419506df9e
parent 18191 ef29685acef0
child 18204 c3caf13f621d
--- a/src/HOL/Isar_examples/Puzzle.thy	Wed Nov 16 17:50:35 2005 +0100
+++ b/src/HOL/Isar_examples/Puzzle.thy	Wed Nov 16 19:34:19 2005 +0100
@@ -4,13 +4,15 @@
 theory Puzzle 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.}
+  \footnote{A question from ``Bundeswettbewerb Mathematik''.  Original
+  pen-and-paper proof due to Herbert Ehler; Isabelle tactic script by
+  Tobias Nipkow.}
+*}
 
- \medskip \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