author | obua |
Sun, 09 May 2004 23:04:36 +0200 | |
changeset 14722 | 8e739a6eaf11 |
parent 14620 | 1be590fd2422 |
child 16417 | 9bc16273c2d4 |
permissions | -rw-r--r-- |
14620
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
1 |
(* Title: HOL/Import/Generate-HOL/GenHOL4Word32.thy |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
2 |
ID: $Id$ |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
3 |
Author: Sebastian Skalberg (TU Muenchen) |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
4 |
*) |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
5 |
|
14516 | 6 |
theory GenHOL4Word32 = GenHOL4Base:; |
7 |
||
8 |
import_segment "hol4"; |
|
9 |
||
10 |
setup_dump "../HOL" "HOL4Word32"; |
|
11 |
||
12 |
append_dump "theory HOL4Word32 = HOL4Base:"; |
|
13 |
||
14 |
import_theory bits; |
|
15 |
||
16 |
const_renames |
|
17 |
BIT > bit |
|
18 |
||
19 |
end_import; |
|
20 |
||
21 |
import_theory word32; |
|
22 |
||
23 |
const_renames |
|
24 |
"==" > EQUIV; |
|
25 |
||
26 |
end_import; |
|
27 |
||
28 |
append_dump "end"; |
|
29 |
||
30 |
flush_dump; |
|
31 |
||
32 |
import_segment ""; |
|
33 |
||
34 |
end |