src/HOL/Isar_examples/Cantor.thy
changeset 7955 f30e08579481
parent 7874 180364256231
child 7982 d534b897ce39
--- a/src/HOL/Isar_examples/Cantor.thy	Wed Oct 27 17:27:07 1999 +0200
+++ b/src/HOL/Isar_examples/Cantor.thy	Wed Oct 27 18:11:54 1999 +0200
@@ -5,8 +5,11 @@
 
 header {* Cantor's Theorem *};
 
-theory Cantor = Main:;text_raw {* \footnote{This is an Isar version of
- the final example of the Isabelle/HOL manual \cite{isabelle-HOL}.}
+theory Cantor = Main:;
+
+text_raw {*
+ \footnote{This is an Isar version of the final example of the
+ Isabelle/HOL manual \cite{isabelle-HOL}.}
 *};
 
 text {*