src/HOL/Algebra/Exponent.thy
changeset 35849 b5522b51cb1e
parent 35848 5443079512ea
child 41413 64cd30d6b0b8
--- a/src/HOL/Algebra/Exponent.thy	Sun Mar 21 16:51:37 2010 +0100
+++ b/src/HOL/Algebra/Exponent.thy	Sun Mar 21 17:12:31 2010 +0100
@@ -1,7 +1,8 @@
 (*  Title:      HOL/Algebra/Exponent.thy
-    Author:     Florian Kammueller, with new proofs by L C Paulson
+    Author:     Florian Kammueller
+    Author:     L C Paulson
 
-    exponent p s   yields the greatest power of p that divides s.
+exponent p s   yields the greatest power of p that divides s.
 *)
 
 theory Exponent