added header
authorkleing
Mon, 20 Aug 2007 04:44:35 +0200
changeset 24334 22863f364531
parent 24333 e77ea0ea7f2c
child 24335 21b4350cf5ec
added header
src/HOL/Word/BitSyntax.thy
--- a/src/HOL/Word/BitSyntax.thy	Mon Aug 20 04:34:31 2007 +0200
+++ b/src/HOL/Word/BitSyntax.thy	Mon Aug 20 04:44:35 2007 +0200
@@ -1,3 +1,11 @@
+(* 
+  ID:     $Id$
+  Author: Brian Huffman, PSU and Gerwin Klein, NICTA
+
+  Syntactic class for bitwise operations.
+*)
+
+
 header {* Syntactic class for bitwise operations *}
 
 theory BitSyntax
@@ -49,10 +57,10 @@
   "bit.B1 OR y = bit.B1"
   "bit.B0 XOR y = y"
   "bit.B1 XOR y = NOT y"
-by (simp_all add: NOT_bit_def AND_bit_def OR_bit_def
-                  XOR_bit_def split: bit.split)
+  by (simp_all add: NOT_bit_def AND_bit_def OR_bit_def
+                    XOR_bit_def split: bit.split)
 
 lemma bit_NOT_NOT: "NOT (NOT (b::bit)) = b"
-by (induct b) simp_all
+  by (induct b) simp_all
 
 end