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
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
24333
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
     1
(* 
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
     2
  ID:     $Id$
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
     3
  Author: Gerwin Klein, NICTA
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
     4
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
     5
  The main interface of the word library to other theories.
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
     6
*)
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
     7
24350
4d74f37c6367 headers for document generation
huffman
parents: 24333
diff changeset
     8
header {* Main Word Library *}
4d74f37c6367 headers for document generation
huffman
parents: 24333
diff changeset
     9
24333
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    10
theory WordMain imports WordGenLib
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    11
begin
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    12
26086
3c243098b64a New simpler representation of numerals, using Bit0 and Bit1 instead of BIT, B0, and B1
huffman
parents: 24350
diff changeset
    13
lemmas word_no_1 [simp] = word_1_no [symmetric, unfolded BIT_simps]
24333
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    14
lemmas word_no_0 [simp] = word_0_no [symmetric]
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    15
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    16
declare word_0_bl [simp]
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    17
declare bin_to_bl_def [simp]
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    18
declare to_bl_0 [simp]
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    19
declare of_bl_True [simp]
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    20
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    21
text "Examples"
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    22
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    23
types word32 = "32 word"
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    24
types word8 = "8 word"
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    25
types byte = word8
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    26
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    27
text {* for more see WordExampes.thy *}
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    28
e77ea0ea7f2c * HOL-Word:
kleing
parents:
diff changeset
    29
end