| author | wenzelm | 
| Thu, 27 Oct 2011 20:26:38 +0200 | |
| changeset 45279 | 89a17197cb98 | 
| parent 44740 | a2940bc24bad | 
| child 46780 | ab4f3f765f91 | 
| permissions | -rw-r--r-- | 
| 14620 
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
 skalberg parents: 
14516diff
changeset | 1 | (* Title: HOL/Import/Generate-HOL/GenHOL4Real.thy | 
| 
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
 skalberg parents: 
14516diff
changeset | 2 | Author: Sebastian Skalberg (TU Muenchen) | 
| 
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
 skalberg parents: 
14516diff
changeset | 3 | *) | 
| 
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
 skalberg parents: 
14516diff
changeset | 4 | |
| 16417 | 5 | theory GenHOL4Real imports GenHOL4Base begin | 
| 14516 | 6 | |
| 7 | import_segment "hol4"; | |
| 8 | ||
| 9 | setup_dump "../HOL" "HOL4Real"; | |
| 10 | ||
| 17566 | 11 | append_dump "theory HOL4Real imports HOL4Base begin"; | 
| 14516 | 12 | |
| 13 | import_theory realax; | |
| 14 | ||
| 15 | type_maps | |
| 16 | real > RealDef.real; | |
| 17 | ||
| 18 | const_maps | |
| 44740 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 19 | real_0 > Groups.zero_class.zero :: real | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 20 | real_1 > Groups.one_class.one :: real | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 21 | real_neg > Groups.uminus_class.uminus :: "real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 22 | inv > Fields.inverse_class.inverse :: "real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 23 | real_add > Groups.plus_class.plus :: "real \<Rightarrow> real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 24 | real_sub > Groups.minus_class.minus :: "real \<Rightarrow> real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 25 | real_mul > Groups.times_class.times :: "real \<Rightarrow> real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 26 | real_div > Fields.inverse_class.divide :: "real \<Rightarrow> real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 27 | real_lt > Orderings.ord_class.less :: "real \<Rightarrow> real \<Rightarrow> bool" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 28 | mk_real > HOL.undefined (* Otherwise proof_import_concl fails *) | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 29 | dest_real > HOL.undefined | 
| 14516 | 30 | |
| 31 | ignore_thms | |
| 32 | real_TY_DEF | |
| 33 | real_tybij | |
| 34 | real_0 | |
| 35 | real_1 | |
| 36 | real_neg | |
| 37 | real_inv | |
| 38 | real_add | |
| 39 | real_mul | |
| 40 | real_lt | |
| 41 | real_of_hreal | |
| 42 | hreal_of_real | |
| 43 | REAL_ISO_EQ | |
| 44 | REAL_POS | |
| 45 | SUP_ALLPOS_LEMMA1 | |
| 46 | SUP_ALLPOS_LEMMA2 | |
| 47 | SUP_ALLPOS_LEMMA3 | |
| 48 | SUP_ALLPOS_LEMMA4; | |
| 49 | ||
| 50 | end_import; | |
| 51 | ||
| 52 | import_theory real; | |
| 53 | ||
| 54 | const_maps | |
| 55 | real_gt > HOL4Compat.real_gt | |
| 56 | real_ge > HOL4Compat.real_ge | |
| 44740 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 57 | real_lte > Orderings.ord_class.less_eq :: "real \<Rightarrow> real \<Rightarrow> bool" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 58 | real_sub > Groups.minus_class.minus :: "real \<Rightarrow> real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 59 | "/" > Fields.inverse_class.divide :: "real \<Rightarrow> real \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 60 | pow > Power.power_class.power :: "real \<Rightarrow> nat \<Rightarrow> real" | 
| 
a2940bc24bad
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
44064diff
changeset | 61 | abs > Groups.abs_class.abs :: "real => real" | 
| 15647 | 62 | real_of_num > RealDef.real :: "nat => real"; | 
| 14516 | 63 | |
| 64 | end_import; | |
| 65 | ||
| 66 | import_theory topology; | |
| 67 | end_import; | |
| 68 | ||
| 69 | import_theory nets; | |
| 70 | end_import; | |
| 71 | ||
| 72 | import_theory seq; | |
| 17694 | 73 | const_renames | 
| 74 | "-->" > "hol4-->"; | |
| 75 | ||
| 14516 | 76 | end_import; | 
| 77 | ||
| 78 | import_theory lim; | |
| 79 | end_import; | |
| 80 | ||
| 81 | import_theory powser; | |
| 82 | end_import; | |
| 83 | ||
| 84 | import_theory transc; | |
| 85 | end_import; | |
| 86 | ||
| 87 | import_theory poly; | |
| 88 | end_import; | |
| 89 | ||
| 90 | append_dump "end"; | |
| 91 | ||
| 92 | flush_dump; | |
| 93 | ||
| 94 | import_segment ""; | |
| 95 | ||
| 96 | end |