src/HOL/Import/Generate-HOLLight/GenHOLLight.thy
author obua
Fri, 16 Sep 2005 21:02:15 +0200
changeset 17440 df77edc4f5d0
parent 17322 781abf7011e6
child 17444 a389e5892691
permissions -rw-r--r--
fixed HOL-light/Isabelle syntax incompatability via more protect_xxx functions

(*  Title:      HOL/Import/Generate-HOLLight/GenHOLLight.thy
    ID:         $Id$
    Author:     Steven Obua (TU Muenchen)
*)

theory GenHOLLight imports "../HOLLightCompat" "../HOL4Syntax" begin;

ML {* reset ProofKernel.debug; *}
ML {* reset Shuffler.debug; *}
ML {* set show_types; set show_sorts; *}

;import_segment "hollight";

setup_dump "../HOLLight" "HOLLight";

append_dump {*theory HOLLight = "../HOLLightCompat" + "../HOL4Syntax":*};

;import_theory hollight;

ignore_thms
  TYDEF_1
  DEF_one
  TYDEF_prod
  TYDEF_num
  IND_SUC_0_EXISTS
  DEF__0
  DEF_SUC
  DEF_IND_SUC
  DEF_IND_0
  DEF_NUM_REP
 (* TYDEF_sum
  DEF_INL
  DEF_INR*);

type_maps
  ind > Nat.ind
  bool > bool
  fun > fun
  N_1 >  Product_Type.unit
  prod > "*"
  num > nat;
 (* sum > "+";*)

const_maps
  T > True
  F > False
  ONE_ONE > HOL4Setup.ONE_ONE
  ONTO    > Fun.surj
  "=" > "op ="
  "==>" > "op -->"
  "/\\" > "op &"
  "\\/" > "op |"
  "!" > All
  "?" > Ex
  "?!" > Ex1
  "~" > Not
  o > Fun.comp
  "@" > "Hilbert_Choice.Eps"
  I > Fun.id
  one > Product_Type.Unity
  LET > HOL4Compat.LET
  mk_pair > Product_Type.Pair_Rep
  "," > Pair
  REP_prod > Rep_Prod
  ABS_prod > Abs_Prod
  FST > fst
  SND > snd
  "_0" > 0 :: nat
  SUC > Suc
  PRE > HOLLightCompat.Pred
  NUMERAL > HOL4Compat.NUMERAL
  "+" > "op +" :: "nat \<Rightarrow> nat \<Rightarrow> nat" 
  "*" > "op *" :: "nat \<Rightarrow> nat \<Rightarrow> nat"
  "-" > "op -" :: "nat \<Rightarrow> nat \<Rightarrow> nat"
  BIT0 > HOLLightCompat.NUMERAL_BIT0
  BIT1 > HOL4Compat.NUMERAL_BIT1;
 (* INL > Sum_Type.Inl
  INR > Sum_Type.Inr
  HAS_SIZE > HOLLightCompat.HAS_SIZE*)

(*import_until "TYDEF_sum"

consts
print_theorems

import_until *)

end_import;

append_dump "end";

flush_dump;

import_segment "";

end