author | haftmann |
Sat, 03 Mar 2012 23:43:21 +0100 | |
changeset 46796 | 81e5ec0a3cd0 |
parent 46787 | 3d3d8f8929a7 |
child 46879 | a8b1236e0837 |
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/GenHOL4Base.thy |
41589 | 2 |
Author: Sebastian Skalberg, TU Muenchen |
14620
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
3 |
*) |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
4 |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
5 |
theory GenHOL4Base |
46796 | 6 |
imports "../../Importer" "../Compatibility" |
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
7 |
begin |
14516 | 8 |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
9 |
import_segment "hol4" |
14516 | 10 |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
11 |
setup_dump "../Generated" "HOL4Base" |
14516 | 12 |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
13 |
append_dump {*theory HOL4Base |
46796 | 14 |
imports "../../Importer" "../Compatibility" |
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
15 |
begin |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
16 |
*} |
14516 | 17 |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
18 |
import_theory "~~/src/HOL/Import/HOL4/Generated" bool; |
14516 | 19 |
|
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:
44377
diff
changeset
|
20 |
type_maps |
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:
44377
diff
changeset
|
21 |
bool > HOL.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:
44377
diff
changeset
|
22 |
|
14516 | 23 |
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:
44377
diff
changeset
|
24 |
T > HOL.True |
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:
44377
diff
changeset
|
25 |
F > HOL.False |
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:
44377
diff
changeset
|
26 |
"!" > HOL.All |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
37678
diff
changeset
|
27 |
"/\\" > HOL.conj |
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
37678
diff
changeset
|
28 |
"\\/" > HOL.disj |
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:
44377
diff
changeset
|
29 |
"?" > HOL.Ex |
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:
44377
diff
changeset
|
30 |
"?!" > HOL.Ex1 |
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:
44377
diff
changeset
|
31 |
"~" > HOL.Not |
17188 | 32 |
COND > HOL.If |
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:
44377
diff
changeset
|
33 |
bool_case > Product_Type.bool.bool_case |
46796 | 34 |
ONE_ONE > Importer.ONE_ONE |
17628 | 35 |
ONTO > Fun.surj |
46796 | 36 |
TYPE_DEFINITION > Importer.TYPE_DEFINITION |
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
37 |
LET > Compatibility.LET; |
14516 | 38 |
|
44377
d3e609c87c4c
reverted some odd changes to HOL/Import (cf. 74c08021ab2e);
wenzelm
parents:
44367
diff
changeset
|
39 |
ignore_thms |
14516 | 40 |
BOUNDED_DEF |
41 |
BOUNDED_THM |
|
42 |
UNBOUNDED_DEF |
|
43 |
UNBOUNDED_THM; |
|
44 |
||
45 |
end_import; |
|
46 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
47 |
import_theory "~~/src/HOL/Import/HOL4/Generated" combin; |
14516 | 48 |
|
49 |
const_maps |
|
50 |
o > Fun.comp; |
|
51 |
||
52 |
end_import; |
|
53 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
54 |
import_theory "~~/src/HOL/Import/HOL4/Generated" sum; |
14516 | 55 |
|
56 |
type_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:
44377
diff
changeset
|
57 |
sum > Sum_Type.sum; |
14516 | 58 |
|
59 |
const_maps |
|
15647 | 60 |
INL > Sum_Type.Inl |
61 |
INR > Sum_Type.Inr |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
62 |
ISL > Compatibility.ISL |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
63 |
ISR > Compatibility.ISR |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
64 |
OUTL > Compatibility.OUTL |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
65 |
OUTR > Compatibility.OUTR |
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:
44377
diff
changeset
|
66 |
sum_case > Sum_Type.sum.sum_case; |
14516 | 67 |
|
68 |
ignore_thms |
|
69 |
sum_TY_DEF |
|
70 |
sum_ISO_DEF |
|
71 |
IS_SUM_REP |
|
72 |
INL_DEF |
|
73 |
INR_DEF |
|
74 |
sum_Axiom; |
|
75 |
||
76 |
end_import; |
|
77 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
78 |
import_theory "~~/src/HOL/Import/HOL4/Generated" one; |
14516 | 79 |
|
80 |
type_maps |
|
81 |
one > Product_Type.unit; |
|
82 |
||
83 |
const_maps |
|
84 |
one > Product_Type.Unity; |
|
85 |
||
86 |
ignore_thms |
|
87 |
one_TY_DEF |
|
88 |
one_axiom |
|
89 |
one_Axiom |
|
90 |
one_DEF; |
|
91 |
||
92 |
end_import; |
|
93 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
94 |
import_theory "~~/src/HOL/Import/HOL4/Generated" option; |
14516 | 95 |
|
96 |
type_maps |
|
30235
58d147683393
Made Option a separate theory and renamed option_map to Option.map
nipkow
parents:
24996
diff
changeset
|
97 |
option > Option.option; |
14516 | 98 |
|
99 |
const_maps |
|
30235
58d147683393
Made Option a separate theory and renamed option_map to Option.map
nipkow
parents:
24996
diff
changeset
|
100 |
NONE > Option.option.None |
58d147683393
Made Option a separate theory and renamed option_map to Option.map
nipkow
parents:
24996
diff
changeset
|
101 |
SOME > Option.option.Some |
58d147683393
Made Option a separate theory and renamed option_map to Option.map
nipkow
parents:
24996
diff
changeset
|
102 |
option_case > Option.option.option_case |
58d147683393
Made Option a separate theory and renamed option_map to Option.map
nipkow
parents:
24996
diff
changeset
|
103 |
OPTION_MAP > Option.map |
58d147683393
Made Option a separate theory and renamed option_map to Option.map
nipkow
parents:
24996
diff
changeset
|
104 |
THE > Option.the |
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
105 |
IS_SOME > Compatibility.IS_SOME |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
106 |
IS_NONE > Compatibility.IS_NONE |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
107 |
OPTION_JOIN > Compatibility.OPTION_JOIN; |
14516 | 108 |
|
109 |
ignore_thms |
|
110 |
option_axiom |
|
111 |
option_Axiom |
|
112 |
option_TY_DEF |
|
113 |
option_REP_ABS_DEF |
|
114 |
SOME_DEF |
|
115 |
NONE_DEF; |
|
116 |
||
117 |
end_import; |
|
118 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
119 |
import_theory "~~/src/HOL/Import/HOL4/Generated" marker; |
14516 | 120 |
end_import; |
121 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
122 |
import_theory "~~/src/HOL/Import/HOL4/Generated" relation; |
14516 | 123 |
|
124 |
const_renames |
|
125 |
reflexive > pred_reflexive; |
|
126 |
||
127 |
end_import; |
|
128 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
129 |
import_theory "~~/src/HOL/Import/HOL4/Generated" pair; |
14516 | 130 |
|
131 |
type_maps |
|
37678
0040bafffdef
"prod" and "sum" replace "*" and "+" respectively
haftmann
parents:
37391
diff
changeset
|
132 |
prod > Product_Type.prod; |
14516 | 133 |
|
134 |
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:
44377
diff
changeset
|
135 |
"," > Product_Type.Pair |
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:
44377
diff
changeset
|
136 |
FST > Product_Type.fst |
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:
44377
diff
changeset
|
137 |
SND > Product_Type.snd |
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:
44377
diff
changeset
|
138 |
CURRY > Product_Type.curry |
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:
44377
diff
changeset
|
139 |
UNCURRY > Product_Type.prod.prod_case |
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:
44377
diff
changeset
|
140 |
"##" > Product_Type.map_pair |
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:
44377
diff
changeset
|
141 |
pair_case > Product_Type.prod.prod_case; |
14516 | 142 |
|
143 |
ignore_thms |
|
144 |
prod_TY_DEF |
|
145 |
MK_PAIR_DEF |
|
146 |
IS_PAIR_DEF |
|
147 |
ABS_REP_prod |
|
148 |
COMMA_DEF; |
|
149 |
||
150 |
end_import; |
|
151 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
152 |
import_theory "~~/src/HOL/Import/HOL4/Generated" num; |
14516 | 153 |
|
154 |
type_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:
44377
diff
changeset
|
155 |
num > Nat.nat; |
14516 | 156 |
|
157 |
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:
44377
diff
changeset
|
158 |
SUC > Nat.Suc |
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:
44377
diff
changeset
|
159 |
0 > Groups.zero_class.zero :: nat; |
14516 | 160 |
|
161 |
ignore_thms |
|
162 |
num_TY_DEF |
|
163 |
num_ISO_DEF |
|
164 |
IS_NUM_REP |
|
165 |
ZERO_REP_DEF |
|
166 |
SUC_REP_DEF |
|
167 |
ZERO_DEF |
|
168 |
SUC_DEF; |
|
169 |
||
170 |
end_import; |
|
171 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
172 |
import_theory "~~/src/HOL/Import/HOL4/Generated" prim_rec; |
14516 | 173 |
|
174 |
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:
44377
diff
changeset
|
175 |
"<" > Orderings.ord_class.less :: "nat \<Rightarrow> nat \<Rightarrow> bool"; |
14516 | 176 |
|
177 |
end_import; |
|
178 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
179 |
import_theory "~~/src/HOL/Import/HOL4/Generated" arithmetic; |
14516 | 180 |
|
181 |
const_maps |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
182 |
ALT_ZERO > Compatibility.ALT_ZERO |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
183 |
NUMERAL_BIT1 > Compatibility.NUMERAL_BIT1 |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
184 |
NUMERAL_BIT2 > Compatibility.NUMERAL_BIT2 |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
185 |
NUMERAL > Compatibility.NUMERAL |
14516 | 186 |
num_case > Nat.nat.nat_case |
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
187 |
">" > Compatibility.nat_gt |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
188 |
">=" > Compatibility.nat_ge |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
189 |
FUNPOW > Compatibility.FUNPOW |
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:
44377
diff
changeset
|
190 |
"<=" > Orderings.ord_class.less_eq :: "nat \<Rightarrow> nat \<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:
44377
diff
changeset
|
191 |
"+" > Groups.plus_class.plus :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
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:
44377
diff
changeset
|
192 |
"*" > Groups.times_class.times :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
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:
44377
diff
changeset
|
193 |
"-" > Groups.minus_class.minus :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
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:
44377
diff
changeset
|
194 |
MIN > Orderings.ord_class.min :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
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:
44377
diff
changeset
|
195 |
MAX > Orderings.ord_class.max :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
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:
44377
diff
changeset
|
196 |
DIV > Divides.div_class.div :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
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:
44377
diff
changeset
|
197 |
MOD > Divides.div_class.mod :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
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:
44377
diff
changeset
|
198 |
EXP > Power.power_class.power :: "nat \<Rightarrow> nat \<Rightarrow> nat"; |
14516 | 199 |
|
200 |
end_import; |
|
201 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
202 |
import_theory "~~/src/HOL/Import/HOL4/Generated" hrat; |
14516 | 203 |
end_import; |
204 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
205 |
import_theory "~~/src/HOL/Import/HOL4/Generated" hreal; |
14516 | 206 |
end_import; |
207 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
208 |
import_theory "~~/src/HOL/Import/HOL4/Generated" numeral; |
14516 | 209 |
end_import; |
210 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
211 |
import_theory "~~/src/HOL/Import/HOL4/Generated" ind_type; |
14516 | 212 |
end_import; |
213 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
214 |
import_theory "~~/src/HOL/Import/HOL4/Generated" divides; |
14516 | 215 |
|
216 |
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:
44377
diff
changeset
|
217 |
divides > Rings.dvd_class.dvd :: "nat \<Rightarrow> nat \<Rightarrow> bool"; |
14516 | 218 |
|
219 |
end_import; |
|
220 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
221 |
import_theory "~~/src/HOL/Import/HOL4/Generated" prime; |
14516 | 222 |
end_import; |
223 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
224 |
import_theory "~~/src/HOL/Import/HOL4/Generated" list; |
14516 | 225 |
|
226 |
type_maps |
|
227 |
list > List.list; |
|
228 |
||
229 |
const_maps |
|
230 |
CONS > List.list.Cons |
|
231 |
NIL > List.list.Nil |
|
232 |
list_case > List.list.list_case |
|
233 |
NULL > List.null |
|
234 |
HD > List.hd |
|
235 |
TL > List.tl |
|
236 |
MAP > List.map |
|
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
237 |
MEM > Compatibility.list_mem |
14516 | 238 |
FILTER > List.filter |
239 |
FOLDL > List.foldl |
|
240 |
EVERY > List.list_all |
|
241 |
REVERSE > List.rev |
|
242 |
LAST > List.last |
|
243 |
FRONT > List.butlast |
|
23029 | 244 |
APPEND > List.append |
14516 | 245 |
FLAT > List.concat |
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:
44377
diff
changeset
|
246 |
LENGTH > Nat.size_class.size |
14516 | 247 |
REPLICATE > List.replicate |
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
248 |
list_size > Compatibility.list_size |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
249 |
SUM > Compatibility.sum |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
250 |
FOLDR > Compatibility.FOLDR |
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:
44377
diff
changeset
|
251 |
EXISTS > List.list_ex |
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
252 |
MAP2 > Compatibility.map2 |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
253 |
ZIP > Compatibility.ZIP |
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
254 |
UNZIP > Compatibility.unzip; |
14516 | 255 |
|
256 |
ignore_thms |
|
257 |
list_TY_DEF |
|
258 |
list_repfns |
|
259 |
list0_def |
|
260 |
list1_def |
|
261 |
NIL |
|
262 |
CONS_def; |
|
263 |
||
264 |
end_import; |
|
265 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
266 |
import_theory "~~/src/HOL/Import/HOL4/Generated" pred_set; |
14516 | 267 |
end_import; |
268 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
269 |
import_theory "~~/src/HOL/Import/HOL4/Generated" operator; |
14516 | 270 |
end_import; |
271 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
272 |
import_theory "~~/src/HOL/Import/HOL4/Generated" rich_list; |
14516 | 273 |
end_import; |
274 |
||
46787
3d3d8f8929a7
file system structure separating HOL4 and HOL Light concerns
haftmann
parents:
46780
diff
changeset
|
275 |
import_theory "~~/src/HOL/Import/HOL4/Generated" state_transformer; |
14516 | 276 |
end_import; |
277 |
||
278 |
append_dump "end"; |
|
279 |
||
280 |
flush_dump; |
|
281 |
||
282 |
import_segment ""; |
|
283 |
||
284 |
end |