src/HOL/Number_Theory/Eratosthenes.thy
changeset 58889 5b7a9633cfa8
parent 58649 a62065b5e1e2
child 60526 fad653acf58f
--- a/src/HOL/Number_Theory/Eratosthenes.thy	Sun Nov 02 18:21:14 2014 +0100
+++ b/src/HOL/Number_Theory/Eratosthenes.thy	Sun Nov 02 18:21:45 2014 +0100
@@ -2,7 +2,7 @@
     Author:     Florian Haftmann, TU Muenchen
 *)
 
-header {* The sieve of Eratosthenes *}
+section {* The sieve of Eratosthenes *}
 
 theory Eratosthenes
 imports Main Primes