src/HOL/Hyperreal/NthRoot.thy
changeset 14767 d2b071e65e4c
parent 14477 cc61fd03e589
child 15085 5693a977a767
--- a/src/HOL/Hyperreal/NthRoot.thy	Fri May 21 21:14:52 2004 +0200
+++ b/src/HOL/Hyperreal/NthRoot.thy	Fri May 21 21:15:10 2004 +0200
@@ -8,10 +8,13 @@
 
 theory NthRoot = SEQ + HSeries:
 
-text{*Various lemmas needed for this result. We follow the proof
-   given by John Lindsay Orr (jorr@math.unl.edu) in his Analysis
-   Webnotes available on the www at http://www.math.unl.edu/~webnotes
-   Lemmas about sequences of reals are used to reach the result.*}
+text {*
+  Various lemmas needed for this result. We follow the proof given by
+  John Lindsay Orr (\texttt{jorr@math.unl.edu}) in his Analysis
+  Webnotes available at \url{http://www.math.unl.edu/~webnotes}.
+
+  Lemmas about sequences of reals are used to reach the result.
+*}
 
 lemma lemma_nth_realpow_non_empty:
      "[| (0::real) < a; 0 < n |] ==> \<exists>s. s : {x. x ^ n <= a & 0 < x}"