| author | wenzelm | 
| Tue, 16 Aug 2005 13:42:47 +0200 | |
| changeset 17076 | c7effdf2e2e2 | 
| parent 16971 | 968adbfbf93b | 
| child 17083 | 051b0897bc98 | 
| permissions | -rw-r--r-- | 
| 923 | 1  | 
(* Title: HOL/hologic.ML  | 
2  | 
ID: $Id$  | 
|
3  | 
Author: Lawrence C Paulson and Markus Wenzel  | 
|
4  | 
||
5  | 
Abstract syntax operations for HOL.  | 
|
6  | 
*)  | 
|
7  | 
||
8  | 
signature HOLOGIC =  | 
|
9  | 
sig  | 
|
| 
12338
 
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
 
wenzelm 
parents: 
11818 
diff
changeset
 | 
10  | 
val typeS: sort  | 
| 
 
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
 
wenzelm 
parents: 
11818 
diff
changeset
 | 
11  | 
val typeT: typ  | 
| 8275 | 12  | 
val boolN: string  | 
| 923 | 13  | 
val boolT: typ  | 
| 7073 | 14  | 
val false_const: term  | 
15  | 
val true_const: term  | 
|
| 923 | 16  | 
val mk_setT: typ -> typ  | 
17  | 
val dest_setT: typ -> typ  | 
|
| 
15965
 
f422f8283491
Use of IntInf.int instead of int in most numeric simprocs; avoids
 
paulson 
parents: 
15945 
diff
changeset
 | 
18  | 
val Trueprop: term  | 
| 923 | 19  | 
val mk_Trueprop: term -> term  | 
20  | 
val dest_Trueprop: term -> term  | 
|
21  | 
val conj: term  | 
|
22  | 
val disj: term  | 
|
23  | 
val imp: term  | 
|
| 8429 | 24  | 
val Not: term  | 
| 7690 | 25  | 
val mk_conj: term * term -> term  | 
26  | 
val mk_disj: term * term -> term  | 
|
27  | 
val mk_imp: term * term -> term  | 
|
| 16835 | 28  | 
val mk_not: term -> term  | 
| 15151 | 29  | 
val dest_conj: term -> term list  | 
| 15945 | 30  | 
val dest_disj: term -> term list  | 
| 4571 | 31  | 
val dest_imp: term -> term * term  | 
| 15151 | 32  | 
val dest_not: term -> term  | 
| 11683 | 33  | 
val dest_concls: term -> term list  | 
| 923 | 34  | 
val eq_const: typ -> term  | 
35  | 
val all_const: typ -> term  | 
|
36  | 
val exists_const: typ -> term  | 
|
| 15945 | 37  | 
val choice_const: typ -> term  | 
| 923 | 38  | 
val Collect_const: typ -> term  | 
39  | 
val mk_eq: term * term -> term  | 
|
| 6031 | 40  | 
val dest_eq: term -> term * term  | 
| 923 | 41  | 
val mk_all: string * typ * term -> term  | 
| 13640 | 42  | 
val list_all: (string * typ) list * term -> term  | 
| 923 | 43  | 
val mk_exists: string * typ * term -> term  | 
44  | 
val mk_Collect: string * typ * term -> term  | 
|
45  | 
val mk_mem: term * term -> term  | 
|
| 6380 | 46  | 
val dest_mem: term -> term * term  | 
| 11818 | 47  | 
val mk_UNIV: typ -> term  | 
| 2510 | 48  | 
val mk_binop: string -> term * term -> term  | 
49  | 
val mk_binrel: string -> term * term -> term  | 
|
50  | 
val dest_bin: string -> typ -> term -> term * term  | 
|
| 4571 | 51  | 
val unitT: typ  | 
| 9362 | 52  | 
val is_unitT: typ -> bool  | 
| 4571 | 53  | 
val unit: term  | 
54  | 
val is_unit: term -> bool  | 
|
55  | 
val mk_prodT: typ * typ -> typ  | 
|
56  | 
val dest_prodT: typ -> typ * typ  | 
|
| 14048 | 57  | 
val pair_const: typ -> typ -> term  | 
| 4571 | 58  | 
val mk_prod: term * term -> term  | 
59  | 
val dest_prod: term -> term * term  | 
|
60  | 
val mk_fst: term -> term  | 
|
61  | 
val mk_snd: term -> term  | 
|
| 
5096
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
62  | 
val prodT_factors: typ -> typ list  | 
| 
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
63  | 
val split_const: typ * typ * typ -> term  | 
| 
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
64  | 
val mk_tuple: typ -> term list -> term  | 
| 5207 | 65  | 
val natT: typ  | 
66  | 
val zero: term  | 
|
67  | 
val is_zero: term -> bool  | 
|
68  | 
val mk_Suc: term -> term  | 
|
69  | 
val dest_Suc: term -> term  | 
|
70  | 
val mk_nat: int -> term  | 
|
71  | 
val dest_nat: term -> int  | 
|
| 7073 | 72  | 
val intT: typ  | 
| 
15965
 
f422f8283491
Use of IntInf.int instead of int in most numeric simprocs; avoids
 
paulson 
parents: 
15945 
diff
changeset
 | 
73  | 
val mk_int: IntInf.int -> term  | 
| 7163 | 74  | 
val realT: typ  | 
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
75  | 
val bitT: typ  | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
76  | 
val B0_const: term  | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
77  | 
val B1_const: term  | 
| 7073 | 78  | 
val binT: typ  | 
79  | 
val pls_const: term  | 
|
80  | 
val min_const: term  | 
|
81  | 
val bit_const: term  | 
|
| 8768 | 82  | 
val number_of_const: typ -> term  | 
| 16971 | 83  | 
val int_of: int list -> IntInf.int  | 
| 
15965
 
f422f8283491
Use of IntInf.int instead of int in most numeric simprocs; avoids
 
paulson 
parents: 
15945 
diff
changeset
 | 
84  | 
val dest_binum: term -> IntInf.int  | 
| 
 
f422f8283491
Use of IntInf.int instead of int in most numeric simprocs; avoids
 
paulson 
parents: 
15945 
diff
changeset
 | 
85  | 
val mk_bin: IntInf.int -> term  | 
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
86  | 
val bin_of : term -> int list  | 
| 13755 | 87  | 
  val mk_list: ('a -> term) -> typ -> 'a list -> term
 | 
| 15062 | 88  | 
val dest_list: term -> term list  | 
| 923 | 89  | 
end;  | 
90  | 
||
| 2510 | 91  | 
|
| 923 | 92  | 
structure HOLogic: HOLOGIC =  | 
93  | 
struct  | 
|
94  | 
||
| 
12338
 
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
 
wenzelm 
parents: 
11818 
diff
changeset
 | 
95  | 
(* HOL syntax *)  | 
| 923 | 96  | 
|
| 
12338
 
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
 
wenzelm 
parents: 
11818 
diff
changeset
 | 
97  | 
val typeS: sort = ["HOL.type"];  | 
| 
 
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
 
wenzelm 
parents: 
11818 
diff
changeset
 | 
98  | 
val typeT = TypeInfer.anyT typeS;  | 
| 
 
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
 
wenzelm 
parents: 
11818 
diff
changeset
 | 
99  | 
|
| 923 | 100  | 
|
| 2510 | 101  | 
(* bool and set *)  | 
| 923 | 102  | 
|
| 8275 | 103  | 
val boolN = "bool";  | 
104  | 
val boolT = Type (boolN, []);  | 
|
| 923 | 105  | 
|
| 9856 | 106  | 
val true_const =  Const ("True", boolT);
 | 
107  | 
val false_const = Const ("False", boolT);
 | 
|
| 7073 | 108  | 
|
| 923 | 109  | 
fun mk_setT T = Type ("set", [T]);
 | 
110  | 
||
111  | 
fun dest_setT (Type ("set", [T])) = T
 | 
|
| 3794 | 112  | 
  | dest_setT T = raise TYPE ("dest_setT: set type expected", [T], []);
 | 
| 923 | 113  | 
|
| 8275 | 114  | 
|
| 7073 | 115  | 
(* logic *)  | 
| 923 | 116  | 
|
117  | 
val Trueprop = Const ("Trueprop", boolT --> propT);
 | 
|
118  | 
||
119  | 
fun mk_Trueprop P = Trueprop $ P;  | 
|
120  | 
||
121  | 
fun dest_Trueprop (Const ("Trueprop", _) $ P) = P
 | 
|
| 3794 | 122  | 
  | dest_Trueprop t = raise TERM ("dest_Trueprop", [t]);
 | 
| 923 | 123  | 
|
124  | 
||
125  | 
val conj = Const ("op &", [boolT, boolT] ---> boolT)
 | 
|
126  | 
and disj = Const ("op |", [boolT, boolT] ---> boolT)
 | 
|
| 8429 | 127  | 
and imp = Const ("op -->", [boolT, boolT] ---> boolT)
 | 
128  | 
and Not = Const ("Not", boolT --> boolT);
 | 
|
| 923 | 129  | 
|
| 7690 | 130  | 
fun mk_conj (t1, t2) = conj $ t1 $ t2  | 
131  | 
and mk_disj (t1, t2) = disj $ t1 $ t2  | 
|
| 16835 | 132  | 
and mk_imp (t1, t2) = imp $ t1 $ t2  | 
133  | 
and mk_not t = Not $ t;  | 
|
| 7690 | 134  | 
|
| 15151 | 135  | 
fun dest_conj (Const ("op &", _) $ t $ t') = t :: dest_conj t'
 | 
136  | 
| dest_conj t = [t];  | 
|
137  | 
||
| 15945 | 138  | 
fun dest_disj (Const ("op |", _) $ t $ t') = t :: dest_disj t'
 | 
139  | 
| dest_disj t = [t];  | 
|
140  | 
||
| 
4466
 
305390f23734
Better equality handling in Blast_tac, usingd a new variant of hyp_subst_tac
 
paulson 
parents: 
4294 
diff
changeset
 | 
141  | 
fun dest_imp (Const("op -->",_) $ A $ B) = (A, B)
 | 
| 
 
305390f23734
Better equality handling in Blast_tac, usingd a new variant of hyp_subst_tac
 
paulson 
parents: 
4294 
diff
changeset
 | 
142  | 
  | dest_imp  t = raise TERM ("dest_imp", [t]);
 | 
| 
 
305390f23734
Better equality handling in Blast_tac, usingd a new variant of hyp_subst_tac
 
paulson 
parents: 
4294 
diff
changeset
 | 
143  | 
|
| 15151 | 144  | 
fun dest_not (Const ("Not", _) $ t) = t
 | 
145  | 
  | dest_not t = raise TERM ("dest_not", [t]);
 | 
|
| 8302 | 146  | 
|
| 11683 | 147  | 
fun imp_concl_of t = imp_concl_of (#2 (dest_imp t)) handle TERM _ => t;  | 
148  | 
val dest_concls = map imp_concl_of o dest_conj o dest_Trueprop;  | 
|
149  | 
||
| 923 | 150  | 
fun eq_const T = Const ("op =", [T, T] ---> boolT);
 | 
151  | 
fun mk_eq (t, u) = eq_const (fastype_of t) $ t $ u;  | 
|
152  | 
||
| 6031 | 153  | 
fun dest_eq (Const ("op =", _) $ lhs $ rhs) = (lhs, rhs)
 | 
154  | 
  | dest_eq t = raise TERM ("dest_eq", [t])
 | 
|
155  | 
||
| 923 | 156  | 
fun all_const T = Const ("All", [T --> boolT] ---> boolT);
 | 
157  | 
fun mk_all (x, T, P) = all_const T $ absfree (x, T, P);  | 
|
| 
15574
 
b1d1b5bfc464
Removed practically all references to Library.foldr.
 
skalberg 
parents: 
15570 
diff
changeset
 | 
158  | 
fun list_all (vs,x) = foldr (fn ((x, T), P) => all_const T $ Abs (x, T, P)) x vs;  | 
| 923 | 159  | 
|
160  | 
fun exists_const T = Const ("Ex", [T --> boolT] ---> boolT);
 | 
|
161  | 
fun mk_exists (x, T, P) = exists_const T $ absfree (x, T, P);  | 
|
162  | 
||
| 15945 | 163  | 
fun choice_const T = Const("Hilbert_Choice.Eps", (T --> boolT) --> T)
 | 
164  | 
||
| 923 | 165  | 
fun Collect_const T = Const ("Collect", [T --> boolT] ---> mk_setT T);
 | 
166  | 
fun mk_Collect (a, T, t) = Collect_const T $ absfree (a, T, t);  | 
|
167  | 
||
168  | 
fun mk_mem (x, A) =  | 
|
169  | 
let val setT = fastype_of A in  | 
|
170  | 
    Const ("op :", [dest_setT setT, setT] ---> boolT) $ x $ A
 | 
|
171  | 
end;  | 
|
172  | 
||
| 6380 | 173  | 
fun dest_mem (Const ("op :", _) $ x $ A) = (x, A)
 | 
174  | 
  | dest_mem t = raise TERM ("dest_mem", [t]);
 | 
|
175  | 
||
| 11818 | 176  | 
fun mk_UNIV T = Const ("UNIV", mk_setT T);
 | 
177  | 
||
| 923 | 178  | 
|
| 
13743
 
f8f9393be64c
Fixed bug in simpdata.ML that prevented the use of congruence rules from a
 
ballarin 
parents: 
13640 
diff
changeset
 | 
179  | 
(* binary operations and relations *)  | 
| 2510 | 180  | 
|
181  | 
fun mk_binop c (t, u) =  | 
|
182  | 
let val T = fastype_of t in  | 
|
183  | 
Const (c, [T, T] ---> T) $ t $ u  | 
|
184  | 
end;  | 
|
185  | 
||
186  | 
fun mk_binrel c (t, u) =  | 
|
187  | 
let val T = fastype_of t in  | 
|
188  | 
Const (c, [T, T] ---> boolT) $ t $ u  | 
|
189  | 
end;  | 
|
190  | 
||
| 
14387
 
e96d5c42c4b0
Polymorphic treatment of binary arithmetic using axclasses
 
paulson 
parents: 
14103 
diff
changeset
 | 
191  | 
(*destruct the application of a binary operator. The dummyT case is a crude  | 
| 
 
e96d5c42c4b0
Polymorphic treatment of binary arithmetic using axclasses
 
paulson 
parents: 
14103 
diff
changeset
 | 
192  | 
way of handling polymorphic operators.*)  | 
| 2510 | 193  | 
fun dest_bin c T (tm as Const (c', Type ("fun", [T', _])) $ t $ u) =
 | 
| 
14387
 
e96d5c42c4b0
Polymorphic treatment of binary arithmetic using axclasses
 
paulson 
parents: 
14103 
diff
changeset
 | 
194  | 
if c = c' andalso (T=T' orelse T=dummyT) then (t, u)  | 
| 3794 | 195  | 
      else raise TERM ("dest_bin " ^ c, [tm])
 | 
196  | 
  | dest_bin c _ tm = raise TERM ("dest_bin " ^ c, [tm]);
 | 
|
| 2510 | 197  | 
|
198  | 
||
| 4571 | 199  | 
(* unit *)  | 
200  | 
||
| 11604 | 201  | 
val unitT = Type ("Product_Type.unit", []);
 | 
| 4571 | 202  | 
|
| 11604 | 203  | 
fun is_unitT (Type ("Product_Type.unit", [])) = true
 | 
| 9362 | 204  | 
| is_unitT _ = false;  | 
205  | 
||
| 11604 | 206  | 
val unit = Const ("Product_Type.Unity", unitT);
 | 
| 4571 | 207  | 
|
| 11604 | 208  | 
fun is_unit (Const ("Product_Type.Unity", _)) = true
 | 
| 4571 | 209  | 
| is_unit _ = false;  | 
210  | 
||
211  | 
||
212  | 
(* prod *)  | 
|
213  | 
||
214  | 
fun mk_prodT (T1, T2) = Type ("*", [T1, T2]);
 | 
|
215  | 
||
216  | 
fun dest_prodT (Type ("*", [T1, T2])) = (T1, T2)
 | 
|
217  | 
  | dest_prodT T = raise TYPE ("dest_prodT", [T], []);
 | 
|
218  | 
||
| 14048 | 219  | 
fun pair_const T1 T2 = Const ("Pair", [T1, T2] ---> mk_prodT (T1, T2));
 | 
220  | 
||
| 4571 | 221  | 
fun mk_prod (t1, t2) =  | 
222  | 
let val T1 = fastype_of t1 and T2 = fastype_of t2 in  | 
|
| 14048 | 223  | 
pair_const T1 T2 $ t1 $ t2  | 
| 4571 | 224  | 
end;  | 
225  | 
||
226  | 
fun dest_prod (Const ("Pair", _) $ t1 $ t2) = (t1, t2)
 | 
|
227  | 
  | dest_prod t = raise TERM ("dest_prod", [t]);
 | 
|
228  | 
||
229  | 
fun mk_fst p =  | 
|
230  | 
let val pT = fastype_of p in  | 
|
231  | 
    Const ("fst", pT --> fst (dest_prodT pT)) $ p
 | 
|
232  | 
end;  | 
|
233  | 
||
234  | 
fun mk_snd p =  | 
|
235  | 
let val pT = fastype_of p in  | 
|
236  | 
    Const ("snd", pT --> snd (dest_prodT pT)) $ p
 | 
|
237  | 
end;  | 
|
238  | 
||
| 
5096
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
239  | 
(*Maps the type T1 * ... * Tn to [T1, ..., Tn], however nested*)  | 
| 
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
240  | 
fun prodT_factors (Type ("*", [T1, T2])) = prodT_factors T1 @ prodT_factors T2
 | 
| 
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
241  | 
| prodT_factors T = [T];  | 
| 
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
242  | 
|
| 16971 | 243  | 
fun split_const (Ta, Tb, Tc) =  | 
| 
5096
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
244  | 
    Const ("split", [[Ta, Tb] ---> Tc, mk_prodT (Ta, Tb)] ---> Tc);
 | 
| 
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
245  | 
|
| 
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
246  | 
(*Makes a nested tuple from a list, following the product type structure*)  | 
| 16971 | 247  | 
fun mk_tuple (Type ("*", [T1, T2])) tms =
 | 
248  | 
mk_prod (mk_tuple T1 tms,  | 
|
| 15570 | 249  | 
mk_tuple T2 (Library.drop (length (prodT_factors T1), tms)))  | 
| 
5096
 
84b00be693b4
Moved most of the Prod_Syntax - stuff to HOLogic.
 
berghofe 
parents: 
4571 
diff
changeset
 | 
250  | 
| mk_tuple T (t::_) = t;  | 
| 4571 | 251  | 
|
| 5207 | 252  | 
|
253  | 
(* nat *)  | 
|
254  | 
||
255  | 
val natT = Type ("nat", []);
 | 
|
256  | 
||
257  | 
val zero = Const ("0", natT);
 | 
|
258  | 
||
259  | 
fun is_zero (Const ("0", _)) = true
 | 
|
260  | 
| is_zero _ = false;  | 
|
261  | 
||
262  | 
fun mk_Suc t = Const ("Suc", natT --> natT) $ t;
 | 
|
263  | 
||
264  | 
fun dest_Suc (Const ("Suc", _) $ t) = t
 | 
|
265  | 
  | dest_Suc t = raise TERM ("dest_Suc", [t]);
 | 
|
266  | 
||
267  | 
fun mk_nat 0 = zero  | 
|
268  | 
| mk_nat n = mk_Suc (mk_nat (n - 1));  | 
|
269  | 
||
270  | 
fun dest_nat (Const ("0", _)) = 0
 | 
|
271  | 
  | dest_nat (Const ("Suc", _) $ t) = dest_nat t + 1
 | 
|
272  | 
  | dest_nat t = raise TERM ("dest_nat", [t]);
 | 
|
273  | 
||
274  | 
||
| 7073 | 275  | 
(* binary numerals *)  | 
276  | 
||
277  | 
val binT = Type ("Numeral.bin", []);
 | 
|
278  | 
||
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
279  | 
val bitT = Type ("Numeral.bit", []);
 | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
280  | 
|
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
281  | 
val B0_const = Const ("Numeral.bit.B0", bitT);
 | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
282  | 
val B1_const =  Const ("Numeral.bit.B1", bitT);
 | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
283  | 
|
| 15013 | 284  | 
val pls_const = Const ("Numeral.Pls", binT)
 | 
285  | 
and min_const = Const ("Numeral.Min", binT)
 | 
|
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
286  | 
and bit_const = Const ("Numeral.Bit", [binT, bitT] ---> binT);
 | 
| 8768 | 287  | 
|
288  | 
fun number_of_const T = Const ("Numeral.number_of", binT --> T);
 | 
|
| 8739 | 289  | 
|
| 16971 | 290  | 
fun int_of [] = 0  | 
| 
15965
 
f422f8283491
Use of IntInf.int instead of int in most numeric simprocs; avoids
 
paulson 
parents: 
15945 
diff
changeset
 | 
291  | 
| int_of (b :: bs) = IntInf.fromInt b + (2 * int_of bs);  | 
| 15595 | 292  | 
|
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
293  | 
(*When called from a print translation, the Numeral qualifier will probably have  | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
294  | 
been removed from Bit, bin.B0, etc.*)  | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
295  | 
fun dest_bit (Const ("Numeral.bit.B0", _)) = 0
 | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
296  | 
  | dest_bit (Const ("Numeral.bit.B1", _)) = 1
 | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
297  | 
  | dest_bit (Const ("bit.B0", _)) = 0
 | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
298  | 
  | dest_bit (Const ("bit.B1", _)) = 1
 | 
| 
7548
 
9e29a3af64ab
ROOT: Integ/bin_simprocs.ML now loaded in Integ/Bin.ML
 
nipkow 
parents: 
7163 
diff
changeset
 | 
299  | 
  | dest_bit t = raise TERM("dest_bit", [t]);
 | 
| 
 
9e29a3af64ab
ROOT: Integ/bin_simprocs.ML now loaded in Integ/Bin.ML
 
nipkow 
parents: 
7163 
diff
changeset
 | 
300  | 
|
| 15013 | 301  | 
fun bin_of (Const ("Numeral.Pls", _)) = []
 | 
302  | 
  | bin_of (Const ("Numeral.Min", _)) = [~1]
 | 
|
303  | 
  | bin_of (Const ("Numeral.Bit", _) $ bs $ b) = dest_bit b :: bin_of bs
 | 
|
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
304  | 
  | bin_of (Const ("Bit", _) $ bs $ b) = dest_bit b :: bin_of bs
 | 
| 
7548
 
9e29a3af64ab
ROOT: Integ/bin_simprocs.ML now loaded in Integ/Bin.ML
 
nipkow 
parents: 
7163 
diff
changeset
 | 
305  | 
  | bin_of t = raise TERM("bin_of", [t]);
 | 
| 
 
9e29a3af64ab
ROOT: Integ/bin_simprocs.ML now loaded in Integ/Bin.ML
 
nipkow 
parents: 
7163 
diff
changeset
 | 
306  | 
|
| 
 
9e29a3af64ab
ROOT: Integ/bin_simprocs.ML now loaded in Integ/Bin.ML
 
nipkow 
parents: 
7163 
diff
changeset
 | 
307  | 
val dest_binum = int_of o bin_of;  | 
| 
 
9e29a3af64ab
ROOT: Integ/bin_simprocs.ML now loaded in Integ/Bin.ML
 
nipkow 
parents: 
7163 
diff
changeset
 | 
308  | 
|
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
309  | 
fun mk_bit 0 = B0_const  | 
| 
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
310  | 
| mk_bit 1 = B1_const  | 
| 10693 | 311  | 
| mk_bit _ = sys_error "mk_bit";  | 
312  | 
||
| 
15965
 
f422f8283491
Use of IntInf.int instead of int in most numeric simprocs; avoids
 
paulson 
parents: 
15945 
diff
changeset
 | 
313  | 
fun mk_bin n =  | 
| 16971 | 314  | 
let  | 
315  | 
fun mk_bit n = if n = 0 then B0_const else B1_const;  | 
|
316  | 
||
317  | 
fun bin_of n =  | 
|
318  | 
if n = 0 then pls_const  | 
|
319  | 
else if n = ~1 then min_const  | 
|
320  | 
else  | 
|
321  | 
let  | 
|
322  | 
(*val (q,r) = IntInf.divMod (n, 2): doesn't work in SML 110.0.7,  | 
|
323  | 
but in newer versions! FIXME: put this back after new SML released!*)  | 
|
324  | 
val q = IntInf.div (n, 2);  | 
|
325  | 
val r = IntInf.mod (n, 2);  | 
|
326  | 
in bit_const $ bin_of q $ mk_bit r end;  | 
|
327  | 
in bin_of n end;  | 
|
| 13755 | 328  | 
|
| 
15620
 
8ccdc8bc66a2
replaced bool by a new datatype "bit" for binary numerals
 
paulson 
parents: 
15595 
diff
changeset
 | 
329  | 
|
| 13755 | 330  | 
(* int *)  | 
331  | 
||
332  | 
val intT = Type ("IntDef.int", []);
 | 
|
333  | 
||
| 
14103
 
afd168fdcd3a
mk_int now produces specific constants for 0 and 1.
 
berghofe 
parents: 
14048 
diff
changeset
 | 
334  | 
fun mk_int 0 = Const ("0", intT)
 | 
| 
 
afd168fdcd3a
mk_int now produces specific constants for 0 and 1.
 
berghofe 
parents: 
14048 
diff
changeset
 | 
335  | 
  | mk_int 1 = Const ("1", intT)
 | 
| 
 
afd168fdcd3a
mk_int now produces specific constants for 0 and 1.
 
berghofe 
parents: 
14048 
diff
changeset
 | 
336  | 
| mk_int i = number_of_const intT $ mk_bin i;  | 
| 13755 | 337  | 
|
338  | 
||
339  | 
(* real *)  | 
|
340  | 
||
| 16971 | 341  | 
val realT = Type ("RealDef.real", []);
 | 
| 13755 | 342  | 
|
343  | 
||
344  | 
(* list *)  | 
|
345  | 
||
346  | 
fun mk_list f T [] = Const ("List.list.Nil", Type ("List.list", [T]))
 | 
|
347  | 
  | mk_list f T (x :: xs) = Const ("List.list.Cons",
 | 
|
348  | 
      T --> Type ("List.list", [T]) --> Type ("List.list", [T])) $ f x $
 | 
|
349  | 
mk_list f T xs;  | 
|
350  | 
||
| 15062 | 351  | 
fun dest_list (Const ("List.list.Nil", _)) = []
 | 
352  | 
  | dest_list (Const ("List.list.Cons", _) $ x $ xs) = x :: dest_list xs
 | 
|
353  | 
  | dest_list t = raise TERM ("dest_list", [t]);
 | 
|
354  | 
||
| 923 | 355  | 
end;  |