src/HOL/Import/Generate-HOL/GenHOL4Word32.thy
author wenzelm
Wed, 31 Aug 2005 15:46:36 +0200
changeset 17199 59c1bfc81d91
parent 16417 9bc16273c2d4
child 17566 484ff733f29c
permissions -rw-r--r--
moved lemmas that require the HOL-Complex logic image to Complex/ex/BigO_Complex.thy; tuned presentation;

(*  Title:      HOL/Import/Generate-HOL/GenHOL4Word32.thy
    ID:         $Id$
    Author:     Sebastian Skalberg (TU Muenchen)
*)

theory GenHOL4Word32 imports GenHOL4Base begin;

import_segment "hol4";

setup_dump "../HOL" "HOL4Word32";

append_dump "theory HOL4Word32 = HOL4Base:";

import_theory bits;

const_renames
  BIT > bit

end_import;

import_theory word32;

const_renames
  "==" > EQUIV;

end_import;

append_dump "end";

flush_dump;

import_segment "";

end