author | wenzelm |
Fri, 20 Mar 2009 15:24:18 +0100 | |
changeset 30607 | c3d1590debd8 |
parent 29269 | 5c25a2012975 |
child 31971 | 8c1b845ed105 |
permissions | -rw-r--r-- |
29269
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
1 |
(* Title: Pure/term_ord.ML |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
2 |
Author: Tobias Nipkow and Makarius, TU Muenchen |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
3 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
4 |
Term orderings. |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
5 |
*) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
6 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
7 |
signature TERM_ORD = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
8 |
sig |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
9 |
val fast_indexname_ord: indexname * indexname -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
10 |
val sort_ord: sort * sort -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
11 |
val typ_ord: typ * typ -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
12 |
val fast_term_ord: term * term -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
13 |
val indexname_ord: indexname * indexname -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
14 |
val tvar_ord: (indexname * sort) * (indexname * sort) -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
15 |
val var_ord: (indexname * typ) * (indexname * typ) -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
16 |
val term_ord: term * term -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
17 |
val hd_ord: term * term -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
18 |
val termless: term * term -> bool |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
19 |
val term_lpo: (term -> int) -> term * term -> order |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
20 |
end; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
21 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
22 |
structure TermOrd: TERM_ORD = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
23 |
struct |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
24 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
25 |
(* fast syntactic ordering -- tuned for inequalities *) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
26 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
27 |
fun fast_indexname_ord ((x, i), (y, j)) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
28 |
(case int_ord (i, j) of EQUAL => fast_string_ord (x, y) | ord => ord); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
29 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
30 |
fun sort_ord SS = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
31 |
if pointer_eq SS then EQUAL |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
32 |
else dict_ord fast_string_ord SS; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
33 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
34 |
local |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
35 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
36 |
fun cons_nr (TVar _) = 0 |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
37 |
| cons_nr (TFree _) = 1 |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
38 |
| cons_nr (Type _) = 2; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
39 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
40 |
in |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
41 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
42 |
fun typ_ord TU = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
43 |
if pointer_eq TU then EQUAL |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
44 |
else |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
45 |
(case TU of |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
46 |
(Type (a, Ts), Type (b, Us)) => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
47 |
(case fast_string_ord (a, b) of EQUAL => dict_ord typ_ord (Ts, Us) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
48 |
| (TFree (a, S), TFree (b, S')) => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
49 |
(case fast_string_ord (a, b) of EQUAL => sort_ord (S, S') | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
50 |
| (TVar (xi, S), TVar (yj, S')) => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
51 |
(case fast_indexname_ord (xi, yj) of EQUAL => sort_ord (S, S') | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
52 |
| (T, U) => int_ord (cons_nr T, cons_nr U)); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
53 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
54 |
end; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
55 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
56 |
local |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
57 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
58 |
fun cons_nr (Const _) = 0 |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
59 |
| cons_nr (Free _) = 1 |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
60 |
| cons_nr (Var _) = 2 |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
61 |
| cons_nr (Bound _) = 3 |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
62 |
| cons_nr (Abs _) = 4 |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
63 |
| cons_nr (_ $ _) = 5; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
64 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
65 |
fun struct_ord (Abs (_, _, t), Abs (_, _, u)) = struct_ord (t, u) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
66 |
| struct_ord (t1 $ t2, u1 $ u2) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
67 |
(case struct_ord (t1, u1) of EQUAL => struct_ord (t2, u2) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
68 |
| struct_ord (t, u) = int_ord (cons_nr t, cons_nr u); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
69 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
70 |
fun atoms_ord (Abs (_, _, t), Abs (_, _, u)) = atoms_ord (t, u) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
71 |
| atoms_ord (t1 $ t2, u1 $ u2) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
72 |
(case atoms_ord (t1, u1) of EQUAL => atoms_ord (t2, u2) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
73 |
| atoms_ord (Const (a, _), Const (b, _)) = fast_string_ord (a, b) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
74 |
| atoms_ord (Free (x, _), Free (y, _)) = fast_string_ord (x, y) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
75 |
| atoms_ord (Var (xi, _), Var (yj, _)) = fast_indexname_ord (xi, yj) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
76 |
| atoms_ord (Bound i, Bound j) = int_ord (i, j) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
77 |
| atoms_ord _ = sys_error "atoms_ord"; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
78 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
79 |
fun types_ord (Abs (_, T, t), Abs (_, U, u)) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
80 |
(case typ_ord (T, U) of EQUAL => types_ord (t, u) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
81 |
| types_ord (t1 $ t2, u1 $ u2) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
82 |
(case types_ord (t1, u1) of EQUAL => types_ord (t2, u2) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
83 |
| types_ord (Const (_, T), Const (_, U)) = typ_ord (T, U) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
84 |
| types_ord (Free (_, T), Free (_, U)) = typ_ord (T, U) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
85 |
| types_ord (Var (_, T), Var (_, U)) = typ_ord (T, U) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
86 |
| types_ord (Bound _, Bound _) = EQUAL |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
87 |
| types_ord _ = sys_error "types_ord"; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
88 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
89 |
in |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
90 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
91 |
fun fast_term_ord tu = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
92 |
if pointer_eq tu then EQUAL |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
93 |
else |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
94 |
(case struct_ord tu of |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
95 |
EQUAL => (case atoms_ord tu of EQUAL => types_ord tu | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
96 |
| ord => ord); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
97 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
98 |
end; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
99 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
100 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
101 |
(* term_ord *) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
102 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
103 |
(*a linear well-founded AC-compatible ordering for terms: |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
104 |
s < t <=> 1. size(s) < size(t) or |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
105 |
2. size(s) = size(t) and s=f(...) and t=g(...) and f<g or |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
106 |
3. size(s) = size(t) and s=f(s1..sn) and t=f(t1..tn) and |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
107 |
(s1..sn) < (t1..tn) (lexicographically)*) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
108 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
109 |
fun indexname_ord ((x, i), (y, j)) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
110 |
(case int_ord (i, j) of EQUAL => string_ord (x, y) | ord => ord); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
111 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
112 |
val tvar_ord = prod_ord indexname_ord sort_ord; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
113 |
val var_ord = prod_ord indexname_ord typ_ord; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
114 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
115 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
116 |
local |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
117 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
118 |
fun hd_depth (t $ _, n) = hd_depth (t, n + 1) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
119 |
| hd_depth p = p; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
120 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
121 |
fun dest_hd (Const (a, T)) = (((a, 0), T), 0) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
122 |
| dest_hd (Free (a, T)) = (((a, 0), T), 1) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
123 |
| dest_hd (Var v) = (v, 2) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
124 |
| dest_hd (Bound i) = ((("", i), dummyT), 3) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
125 |
| dest_hd (Abs (_, T, _)) = ((("", 0), T), 4); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
126 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
127 |
in |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
128 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
129 |
fun term_ord tu = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
130 |
if pointer_eq tu then EQUAL |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
131 |
else |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
132 |
(case tu of |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
133 |
(Abs (_, T, t), Abs(_, U, u)) => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
134 |
(case term_ord (t, u) of EQUAL => typ_ord (T, U) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
135 |
| (t, u) => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
136 |
(case int_ord (size_of_term t, size_of_term u) of |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
137 |
EQUAL => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
138 |
(case prod_ord hd_ord int_ord (hd_depth (t, 0), hd_depth (u, 0)) of |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
139 |
EQUAL => args_ord (t, u) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
140 |
| ord => ord)) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
141 |
and hd_ord (f, g) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
142 |
prod_ord (prod_ord indexname_ord typ_ord) int_ord (dest_hd f, dest_hd g) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
143 |
and args_ord (f $ t, g $ u) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
144 |
(case args_ord (f, g) of EQUAL => term_ord (t, u) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
145 |
| args_ord _ = EQUAL; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
146 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
147 |
fun termless tu = (term_ord tu = LESS); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
148 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
149 |
end; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
150 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
151 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
152 |
(* Lexicographic path order on terms *) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
153 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
154 |
(* |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
155 |
See Baader & Nipkow, Term rewriting, CUP 1998. |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
156 |
Without variables. Const, Var, Bound, Free and Abs are treated all as |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
157 |
constants. |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
158 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
159 |
f_ord maps terms to integers and serves two purposes: |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
160 |
- Predicate on constant symbols. Those that are not recognised by f_ord |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
161 |
must be mapped to ~1. |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
162 |
- Order on the recognised symbols. These must be mapped to distinct |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
163 |
integers >= 0. |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
164 |
The argument of f_ord is never an application. |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
165 |
*) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
166 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
167 |
local |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
168 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
169 |
fun unrecognized (Const (a, T)) = ((1, ((a, 0), T)), 0) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
170 |
| unrecognized (Free (a, T)) = ((1, ((a, 0), T)), 0) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
171 |
| unrecognized (Var v) = ((1, v), 1) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
172 |
| unrecognized (Bound i) = ((1, (("", i), dummyT)), 2) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
173 |
| unrecognized (Abs (_, T, _)) = ((1, (("", 0), T)), 3); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
174 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
175 |
fun dest_hd f_ord t = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
176 |
let val ord = f_ord t |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
177 |
in if ord = ~1 then unrecognized t else ((0, (("", ord), fastype_of t)), 0) end; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
178 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
179 |
fun term_lpo f_ord (s, t) = |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
180 |
let val (f, ss) = strip_comb s and (g, ts) = strip_comb t in |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
181 |
if forall (fn si => term_lpo f_ord (si, t) = LESS) ss |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
182 |
then case hd_ord f_ord (f, g) of |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
183 |
GREATER => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
184 |
if forall (fn ti => term_lpo f_ord (s, ti) = GREATER) ts |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
185 |
then GREATER else LESS |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
186 |
| EQUAL => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
187 |
if forall (fn ti => term_lpo f_ord (s, ti) = GREATER) ts |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
188 |
then list_ord (term_lpo f_ord) (ss, ts) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
189 |
else LESS |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
190 |
| LESS => LESS |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
191 |
else GREATER |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
192 |
end |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
193 |
and hd_ord f_ord (f, g) = case (f, g) of |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
194 |
(Abs (_, T, t), Abs (_, U, u)) => |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
195 |
(case term_lpo f_ord (t, u) of EQUAL => typ_ord (T, U) | ord => ord) |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
196 |
| (_, _) => prod_ord (prod_ord int_ord |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
197 |
(prod_ord indexname_ord typ_ord)) int_ord |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
198 |
(dest_hd f_ord f, dest_hd f_ord g); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
199 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
200 |
in |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
201 |
val term_lpo = term_lpo |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
202 |
end; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
203 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
204 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
205 |
end; |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
206 |
|
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
207 |
structure Vartab = TableFun(type key = indexname val ord = TermOrd.fast_indexname_ord); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
208 |
structure Typtab = TableFun(type key = typ val ord = TermOrd.typ_ord); |
5c25a2012975
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
wenzelm
parents:
diff
changeset
|
209 |
structure Termtab = TableFun(type key = term val ord = TermOrd.fast_term_ord); |