src/ZF/Bin.thy
changeset 58871 c399ae4b836f
parent 58421 37cbbd8eb460
child 59748 a1c35e6fe735
--- a/src/ZF/Bin.thy	Sun Nov 02 16:09:35 2014 +0100
+++ b/src/ZF/Bin.thy	Sun Nov 02 16:39:54 2014 +0100
@@ -13,7 +13,7 @@
 For instance, ~5 div 2 = ~3 and ~5 mod 2 = 1; thus ~5 = (~3)*2 + 1
 *)
 
-header{*Arithmetic on Binary Integers*}
+section{*Arithmetic on Binary Integers*}
 
 theory Bin
 imports Int_ZF Datatype_ZF