src/HOL/Algebra/Exponent.thy
changeset 20318 0e0ea63fe768
parent 20282 49c312eaaa11
child 20432 07ec57376051
--- a/src/HOL/Algebra/Exponent.thy	Thu Aug 03 14:53:57 2006 +0200
+++ b/src/HOL/Algebra/Exponent.thy	Thu Aug 03 14:57:26 2006 +0200
@@ -5,14 +5,15 @@
     exponent p s   yields the greatest power of p that divides s.
 *)
 
-header{*The Combinatorial Argument Underlying the First Sylow Theorem*}
-
 theory Exponent imports Main Primes begin
 
+
+section {*The Combinatorial Argument Underlying the First Sylow Theorem*}
 constdefs
   exponent      :: "[nat, nat] => nat"
   "exponent p s == if prime p then (GREATEST r. p^r dvd s) else 0"
 
+
 subsection{*Prime Theorems*}
 
 lemma prime_imp_one_less: "prime p ==> Suc 0 < p"
@@ -196,7 +197,7 @@
 done
 
 
-subsection{*Lemmas for the Main Combinatorial Argument*}
+subsection{*Main Combinatorial Argument*}
 
 lemma le_extend_mult: "[| 0 < c; a <= b |] ==> a <= b * (c::nat)"
 apply (rule_tac P = "%x. x <= b * c" in subst)