src/HOL/ex/Birthday_Paradox.thy
changeset 58889 5b7a9633cfa8
parent 50123 69b35a75caf3
child 59669 de7792ea4090
--- a/src/HOL/ex/Birthday_Paradox.thy	Sun Nov 02 18:21:14 2014 +0100
+++ b/src/HOL/ex/Birthday_Paradox.thy	Sun Nov 02 18:21:45 2014 +0100
@@ -2,7 +2,7 @@
     Author: Lukas Bulwahn, TU Muenchen, 2007
 *)
 
-header {* A Formulation of the Birthday Paradox *}
+section {* A Formulation of the Birthday Paradox *}
 
 theory Birthday_Paradox
 imports Main "~~/src/HOL/Fact" "~~/src/HOL/Library/FuncSet"