diff -r ed47044ee6a6 -r 2e48182cc82c src/HOL/Isar_Examples/Puzzle.thy --- a/src/HOL/Isar_Examples/Puzzle.thy Sat Dec 26 15:03:41 2015 +0100 +++ b/src/HOL/Isar_Examples/Puzzle.thy Sat Dec 26 15:44:14 2015 +0100 @@ -4,12 +4,14 @@ 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 \\<^bold>\Problem.\ Given some function \f: \ \ \\ such that - \f (f n) < f (Suc n)\ for all \n\. Demonstrate that \f\ is the identity.\ +text \ + \<^bold>\Problem.\ Given some function \f: \ \ \\ such that \f (f n) < f (Suc n)\ + for all \n\. Demonstrate that \f\ is the identity. +\ theorem assumes f_ax: "\n. f (f n) < f (Suc n)"