src/HOL/Word/BinGeneral.thy
changeset 24350 4d74f37c6367
parent 24333 e77ea0ea7f2c
child 24364 31e359126ab6
--- a/src/HOL/Word/BinGeneral.thy	Mon Aug 20 18:10:13 2007 +0200
+++ b/src/HOL/Word/BinGeneral.thy	Mon Aug 20 18:11:09 2007 +0200
@@ -7,10 +7,14 @@
   in particular, bin_rec and related work
 *) 
 
+header {* Basic Definitions for Binary Integers *}
+
 theory BinGeneral imports TdThs Num_Lemmas
 
 begin
 
+subsection {* Recursion combinator for binary integers *}
+
 lemma brlem: "(bin = Numeral.Min) = (- bin + Numeral.pred 0 = 0)"
   unfolding Min_def pred_def by arith
 
@@ -299,7 +303,7 @@
   by (auto simp: pred_def succ_def split add : split_if_asm)
 
 
-section "Simplifications for (s)bintrunc"
+subsection "Simplifications for (s)bintrunc"
 
 lemma bit_bool:
   "(b = (b' = bit.B1)) = (b' = (if b then bit.B1 else bit.B0))"