author | wenzelm |
Sun, 21 Dec 2014 19:14:16 +0100 | |
changeset 59169 | ddc948e4ed09 |
parent 58881 | b9556a055632 |
child 59582 | 0fbed69ff081 |
permissions | -rw-r--r-- |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
1 |
(* Title: HOL/Library/Code_Abstract_Nat.thy |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
2 |
Author: Stefan Berghofer, Florian Haftmann, TU Muenchen |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
3 |
*) |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
4 |
|
58881 | 5 |
section {* Avoidance of pattern matching on natural numbers *} |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
6 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
7 |
theory Code_Abstract_Nat |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
8 |
imports Main |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
9 |
begin |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
10 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
11 |
text {* |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
12 |
When natural numbers are implemented in another than the |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
13 |
conventional inductive @{term "0::nat"}/@{term Suc} representation, |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
14 |
it is necessary to avoid all pattern matching on natural numbers |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
15 |
altogether. This is accomplished by this theory (up to a certain |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
16 |
extent). |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
17 |
*} |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
18 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
19 |
subsection {* Case analysis *} |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
20 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
21 |
text {* |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
22 |
Case analysis on natural numbers is rephrased using a conditional |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
23 |
expression: |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
24 |
*} |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
25 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
26 |
lemma [code, code_unfold]: |
55415 | 27 |
"case_nat = (\<lambda>f g n. if n = 0 then f else g (n - 1))" |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
28 |
by (auto simp add: fun_eq_iff dest!: gr0_implies_Suc) |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
29 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
30 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
31 |
subsection {* Preprocessors *} |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
32 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
33 |
text {* |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
34 |
The term @{term "Suc n"} is no longer a valid pattern. Therefore, |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
35 |
all occurrences of this term in a position where a pattern is |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
36 |
expected (i.e.~on the left-hand side of a code equation) must be |
56790
f54097170704
prefer plain ASCII / latex over not-so-universal Unicode;
wenzelm
parents:
55757
diff
changeset
|
37 |
eliminated. This can be accomplished -- as far as possible -- by |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
38 |
applying the following transformation rule: |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
39 |
*} |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
40 |
|
57426 | 41 |
lemma Suc_if_eq: |
42 |
assumes "\<And>n. f (Suc n) \<equiv> h n" |
|
43 |
assumes "f 0 \<equiv> g" |
|
44 |
shows "f n \<equiv> if n = 0 then g else h (n - 1)" |
|
45 |
by (rule eq_reflection) (cases n, insert assms, simp_all) |
|
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
46 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
47 |
text {* |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
48 |
The rule above is built into a preprocessor that is plugged into |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
49 |
the code generator. |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
50 |
*} |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
51 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
52 |
setup {* |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
53 |
let |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
54 |
|
57427 | 55 |
val Suc_if_eq = Thm.incr_indexes 1 @{thm Suc_if_eq}; |
56 |
||
55757 | 57 |
fun remove_suc ctxt thms = |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
58 |
let |
55757 | 59 |
val thy = Proof_Context.theory_of ctxt; |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
60 |
val vname = singleton (Name.variant_list (map fst |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
61 |
(fold (Term.add_var_names o Thm.full_prop_of) thms []))) "n"; |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
62 |
val cv = cterm_of thy (Var ((vname, 0), HOLogic.natT)); |
57426 | 63 |
val lhs_of = snd o Thm.dest_comb o fst o Thm.dest_comb o cprop_of; |
64 |
val rhs_of = snd o Thm.dest_comb o cprop_of; |
|
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
65 |
fun find_vars ct = (case term_of ct of |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
66 |
(Const (@{const_name Suc}, _) $ Var _) => [(cv, snd (Thm.dest_comb ct))] |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
67 |
| _ $ _ => |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
68 |
let val (ct1, ct2) = Thm.dest_comb ct |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
69 |
in |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
70 |
map (apfst (fn ct => Thm.apply ct ct2)) (find_vars ct1) @ |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
71 |
map (apfst (Thm.apply ct1)) (find_vars ct2) |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
72 |
end |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
73 |
| _ => []); |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
74 |
val eqs = maps |
57426 | 75 |
(fn thm => map (pair thm) (find_vars (lhs_of thm))) thms; |
76 |
fun mk_thms (thm, (ct, cv')) = |
|
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
77 |
let |
57426 | 78 |
val thm' = |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
79 |
Thm.implies_elim |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
80 |
(Conv.fconv_rule (Thm.beta_conversion true) |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
81 |
(Drule.instantiate' |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
82 |
[SOME (ctyp_of_term ct)] [SOME (Thm.lambda cv ct), |
57426 | 83 |
SOME (Thm.lambda cv' (rhs_of thm)), NONE, SOME cv'] |
57427 | 84 |
Suc_if_eq)) (Thm.forall_intr cv' thm) |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
85 |
in |
57426 | 86 |
case map_filter (fn thm'' => |
87 |
SOME (thm'', singleton |
|
88 |
(Variable.trade (K (fn [thm'''] => [thm''' RS thm'])) |
|
59169 | 89 |
(Variable.declare_thm thm'' ctxt)) thm'') |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
90 |
handle THM _ => NONE) thms of |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
91 |
[] => NONE |
57426 | 92 |
| thmps => |
93 |
let val (thms1, thms2) = split_list thmps |
|
94 |
in SOME (subtract Thm.eq_thm (thm :: thms1) thms @ thms2) end |
|
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
95 |
end |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
96 |
in get_first mk_thms eqs end; |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
97 |
|
59169 | 98 |
fun eqn_suc_base_preproc ctxt thms = |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
99 |
let |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
100 |
val dest = fst o Logic.dest_equals o prop_of; |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
101 |
val contains_suc = exists_Const (fn (c, _) => c = @{const_name Suc}); |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
102 |
in |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
103 |
if forall (can dest) thms andalso exists (contains_suc o dest) thms |
59169 | 104 |
then thms |> perhaps_loop (remove_suc ctxt) |> (Option.map o map) Drule.zero_var_indexes |
51113
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
105 |
else NONE |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
106 |
end; |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
107 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
108 |
val eqn_suc_preproc = Code_Preproc.simple_functrans eqn_suc_base_preproc; |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
109 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
110 |
in |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
111 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
112 |
Code_Preproc.add_functrans ("eqn_Suc", eqn_suc_preproc) |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
113 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
114 |
end; |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
115 |
*} |
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
116 |
|
222fb6cb2c3e
factored out shared preprocessor setup into theory Code_Abstract_Nat, tuning descriptions
haftmann
parents:
diff
changeset
|
117 |
end |