diff -r 27f3c10b0b50 -r 4cf66f21b764 src/HOL/Word/Bits.thy --- a/src/HOL/Word/Bits.thy Mon Dec 07 10:23:50 2015 +0100 +++ b/src/HOL/Word/Bits.thy Mon Dec 07 10:38:04 2015 +0100 @@ -2,7 +2,7 @@ Author: Author: Brian Huffman, PSU and Gerwin Klein, NICTA *) -section {* Syntactic classes for bitwise operations *} +section \Syntactic classes for bitwise operations\ theory Bits imports Main @@ -14,15 +14,15 @@ and bitOR :: "'a \ 'a \ 'a" (infixr "OR" 59) and bitXOR :: "'a \ 'a \ 'a" (infixr "XOR" 59) -text {* +text \ We want the bitwise operations to bind slightly weaker - than @{text "+"} and @{text "-"}, but @{text "~~"} to - bind slightly stronger than @{text "*"}. -*} + than \+\ and \-\, but \~~\ to + bind slightly stronger than \*\. +\ -text {* +text \ Testing and shifting operations. -*} +\ class bits = bit + fixes test_bit :: "'a \ nat \ bool" (infixl "!!" 100)