src/HOL/Import/Generate-HOL/GenHOL4Vec.thy
author haftmann
Fri, 24 Feb 2012 22:46:44 +0100
changeset 46664 1f6c140f9c72
parent 41589 bbd861837ebc
child 46780 ab4f3f765f91
permissions -rw-r--r--
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy

(*  Title:      HOL/Import/Generate-HOL/GenHOL4Vec.thy
    Author:     Sebastian Skalberg, TU Muenchen
*)

theory GenHOL4Vec imports GenHOL4Base begin

import_segment "hol4";

setup_dump "../HOL" "HOL4Vec";

append_dump "theory HOL4Vec imports HOL4Base begin";

import_theory res_quan;
end_import;

import_theory word_base;

const_renames
  BIT > bit;

end_import;

import_theory word_num;
end_import;

import_theory word_bitop;
end_import;

import_theory bword_num;
end_import;

import_theory bword_arith;
end_import;

import_theory bword_bitop;
end_import;

append_dump "end";

flush_dump;

import_segment "";

end