src/HOL/Word/Bit_Operations.thy
changeset 53062 3af1a6020014
parent 41413 64cd30d6b0b8
child 53438 6301ed01e34d
--- a/src/HOL/Word/Bit_Operations.thy	Sun Aug 18 13:58:33 2013 +0200
+++ b/src/HOL/Word/Bit_Operations.thy	Sun Aug 18 15:29:50 2013 +0200
@@ -8,6 +8,8 @@
 imports "~~/src/HOL/Library/Bit"
 begin
 
+subsection {* Abstract syntactic bit operations *}
+
 class bit =
   fixes bitNOT :: "'a \<Rightarrow> 'a"       ("NOT _" [70] 71)
     and bitAND :: "'a \<Rightarrow> 'a \<Rightarrow> 'a" (infixr "AND" 64)
@@ -35,7 +37,7 @@
 class bitss = bits +
   fixes msb      :: "'a \<Rightarrow> bool"
 
-
+  
 subsection {* Bitwise operations on @{typ bit} *}
 
 instantiation bit :: bit