src/HOL/Word/WordMain.thy
author huffman
Sun, 17 Feb 2008 06:49:53 +0100
changeset 26086 3c243098b64a
parent 24350 4d74f37c6367
child 26560 d2fc9a18ee8a
permissions -rw-r--r--
New simpler representation of numerals, using Bit0 and Bit1 instead of BIT, B0, and B1

(* 
  ID:     $Id$
  Author: Gerwin Klein, NICTA

  The main interface of the word library to other theories.
*)

header {* Main Word Library *}

theory WordMain imports WordGenLib
begin

lemmas word_no_1 [simp] = word_1_no [symmetric, unfolded BIT_simps]
lemmas word_no_0 [simp] = word_0_no [symmetric]

declare word_0_bl [simp]
declare bin_to_bl_def [simp]
declare to_bl_0 [simp]
declare of_bl_True [simp]

text "Examples"

types word32 = "32 word"
types word8 = "8 word"
types byte = word8

text {* for more see WordExampes.thy *}

end