author | wenzelm |
Sat, 20 Oct 2012 15:46:48 +0200 | |
changeset 49954 | 44658062d822 |
parent 49950 | cd882d53ba6b |
child 49972 | f11f8905d9fd |
permissions | -rw-r--r-- |
31596 | 1 |
(* Author: Florian Haftmann, TU Muenchen *) |
26348 | 2 |
|
3 |
header {* Finite types as explicit enumerations *} |
|
4 |
||
5 |
theory Enum |
|
40650
d40b347d5b0b
adding Enum to HOL-Main image and removing it from HOL-Library
bulwahn
parents:
40649
diff
changeset
|
6 |
imports Map String |
26348 | 7 |
begin |
8 |
||
9 |
subsection {* Class @{text enum} *} |
|
10 |
||
29797 | 11 |
class enum = |
26348 | 12 |
fixes enum :: "'a list" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
13 |
fixes enum_all :: "('a \<Rightarrow> bool) \<Rightarrow> bool" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
14 |
fixes enum_ex :: "('a \<Rightarrow> bool) \<Rightarrow> bool" |
33635 | 15 |
assumes UNIV_enum: "UNIV = set enum" |
26444 | 16 |
and enum_distinct: "distinct enum" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
17 |
assumes enum_all_UNIV: "enum_all P \<longleftrightarrow> Ball UNIV P" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
18 |
assumes enum_ex_UNIV: "enum_ex P \<longleftrightarrow> Bex UNIV P" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
19 |
-- {* tailored towards simple instantiation *} |
26348 | 20 |
begin |
21 |
||
29797 | 22 |
subclass finite proof |
23 |
qed (simp add: UNIV_enum) |
|
26444 | 24 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
25 |
lemma enum_UNIV: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
26 |
"set enum = UNIV" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
27 |
by (simp only: UNIV_enum) |
26444 | 28 |
|
40683 | 29 |
lemma in_enum: "x \<in> set enum" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
30 |
by (simp add: enum_UNIV) |
26348 | 31 |
|
32 |
lemma enum_eq_I: |
|
33 |
assumes "\<And>x. x \<in> set xs" |
|
34 |
shows "set enum = set xs" |
|
35 |
proof - |
|
36 |
from assms UNIV_eq_I have "UNIV = set xs" by auto |
|
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
37 |
with enum_UNIV show ?thesis by simp |
26348 | 38 |
qed |
39 |
||
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
40 |
lemma enum_all [simp]: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
41 |
"enum_all = HOL.All" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
42 |
by (simp add: fun_eq_iff enum_all_UNIV) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
43 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
44 |
lemma enum_ex [simp]: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
45 |
"enum_ex = HOL.Ex" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
46 |
by (simp add: fun_eq_iff enum_ex_UNIV) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
47 |
|
26348 | 48 |
end |
49 |
||
50 |
||
49949 | 51 |
subsection {* Implementations using @{class enum} *} |
52 |
||
53 |
subsubsection {* Unbounded operations and quantifiers *} |
|
54 |
||
55 |
lemma Collect_code [code]: |
|
56 |
"Collect P = set (filter P enum)" |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
57 |
by (simp add: enum_UNIV) |
49949 | 58 |
|
59 |
definition card_UNIV :: "'a itself \<Rightarrow> nat" |
|
60 |
where |
|
61 |
[code del]: "card_UNIV TYPE('a) = card (UNIV :: 'a set)" |
|
62 |
||
63 |
lemma [code]: |
|
64 |
"card_UNIV TYPE('a :: enum) = card (set (Enum.enum :: 'a list))" |
|
65 |
by (simp only: card_UNIV_def enum_UNIV) |
|
66 |
||
67 |
lemma all_code [code]: "(\<forall>x. P x) \<longleftrightarrow> enum_all P" |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
68 |
by simp |
49949 | 69 |
|
70 |
lemma exists_code [code]: "(\<exists>x. P x) \<longleftrightarrow> enum_ex P" |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
71 |
by simp |
49949 | 72 |
|
73 |
lemma exists1_code [code]: "(\<exists>!x. P x) \<longleftrightarrow> list_ex1 P enum" |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
74 |
by (auto simp add: list_ex1_iff enum_UNIV) |
49949 | 75 |
|
76 |
||
77 |
subsubsection {* An executable choice operator *} |
|
78 |
||
79 |
definition |
|
80 |
[code del]: "enum_the = The" |
|
81 |
||
82 |
lemma [code]: |
|
83 |
"The P = (case filter P enum of [x] => x | _ => enum_the P)" |
|
84 |
proof - |
|
85 |
{ |
|
86 |
fix a |
|
87 |
assume filter_enum: "filter P enum = [a]" |
|
88 |
have "The P = a" |
|
89 |
proof (rule the_equality) |
|
90 |
fix x |
|
91 |
assume "P x" |
|
92 |
show "x = a" |
|
93 |
proof (rule ccontr) |
|
94 |
assume "x \<noteq> a" |
|
95 |
from filter_enum obtain us vs |
|
96 |
where enum_eq: "enum = us @ [a] @ vs" |
|
97 |
and "\<forall> x \<in> set us. \<not> P x" |
|
98 |
and "\<forall> x \<in> set vs. \<not> P x" |
|
99 |
and "P a" |
|
100 |
by (auto simp add: filter_eq_Cons_iff) (simp only: filter_empty_conv[symmetric]) |
|
101 |
with `P x` in_enum[of x, unfolded enum_eq] `x \<noteq> a` show "False" by auto |
|
102 |
qed |
|
103 |
next |
|
104 |
from filter_enum show "P a" by (auto simp add: filter_eq_Cons_iff) |
|
105 |
qed |
|
106 |
} |
|
107 |
from this show ?thesis |
|
108 |
unfolding enum_the_def by (auto split: list.split) |
|
109 |
qed |
|
110 |
||
111 |
code_abort enum_the |
|
112 |
code_const enum_the (Eval "(fn p => raise Match)") |
|
113 |
||
114 |
||
115 |
subsubsection {* Equality and order on functions *} |
|
26348 | 116 |
|
38857
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
haftmann
parents:
37765
diff
changeset
|
117 |
instantiation "fun" :: (enum, equal) equal |
26513 | 118 |
begin |
26348 | 119 |
|
26513 | 120 |
definition |
38857
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
haftmann
parents:
37765
diff
changeset
|
121 |
"HOL.equal f g \<longleftrightarrow> (\<forall>x \<in> set enum. f x = g x)" |
26513 | 122 |
|
31464 | 123 |
instance proof |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
124 |
qed (simp_all add: equal_fun_def fun_eq_iff enum_UNIV) |
26513 | 125 |
|
126 |
end |
|
26348 | 127 |
|
40898
882e860a1e83
changed order of lemmas to overwrite the general code equation with the nbe-specific one
bulwahn
parents:
40683
diff
changeset
|
128 |
lemma [code]: |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
129 |
"HOL.equal f g \<longleftrightarrow> enum_all (%x. f x = g x)" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
130 |
by (auto simp add: equal fun_eq_iff) |
40898
882e860a1e83
changed order of lemmas to overwrite the general code equation with the nbe-specific one
bulwahn
parents:
40683
diff
changeset
|
131 |
|
38857
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
haftmann
parents:
37765
diff
changeset
|
132 |
lemma [code nbe]: |
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
haftmann
parents:
37765
diff
changeset
|
133 |
"HOL.equal (f :: _ \<Rightarrow> _) f \<longleftrightarrow> True" |
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
haftmann
parents:
37765
diff
changeset
|
134 |
by (fact equal_refl) |
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
haftmann
parents:
37765
diff
changeset
|
135 |
|
28562 | 136 |
lemma order_fun [code]: |
26348 | 137 |
fixes f g :: "'a\<Colon>enum \<Rightarrow> 'b\<Colon>order" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
138 |
shows "f \<le> g \<longleftrightarrow> enum_all (\<lambda>x. f x \<le> g x)" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
139 |
and "f < g \<longleftrightarrow> f \<le> g \<and> enum_ex (\<lambda>x. f x \<noteq> g x)" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
140 |
by (simp_all add: fun_eq_iff le_fun_def order_less_le) |
26968 | 141 |
|
142 |
||
49949 | 143 |
subsubsection {* Operations on relations *} |
144 |
||
145 |
lemma [code]: |
|
146 |
"Id = image (\<lambda>x. (x, x)) (set Enum.enum)" |
|
147 |
by (auto intro: imageI in_enum) |
|
26968 | 148 |
|
49949 | 149 |
lemma tranclp_unfold [code, no_atp]: |
150 |
"tranclp r a b \<longleftrightarrow> (a, b) \<in> trancl {(x, y). r x y}" |
|
151 |
by (simp add: trancl_def) |
|
152 |
||
153 |
lemma rtranclp_rtrancl_eq [code, no_atp]: |
|
154 |
"rtranclp r x y \<longleftrightarrow> (x, y) \<in> rtrancl {(x, y). r x y}" |
|
155 |
by (simp add: rtrancl_def) |
|
26968 | 156 |
|
49949 | 157 |
lemma max_ext_eq [code]: |
158 |
"max_ext R = {(X, Y). finite X \<and> finite Y \<and> Y \<noteq> {} \<and> (\<forall>x. x \<in> X \<longrightarrow> (\<exists>xa \<in> Y. (x, xa) \<in> R))}" |
|
159 |
by (auto simp add: max_ext.simps) |
|
160 |
||
161 |
lemma max_extp_eq [code]: |
|
162 |
"max_extp r x y \<longleftrightarrow> (x, y) \<in> max_ext {(x, y). r x y}" |
|
163 |
by (simp add: max_ext_def) |
|
26348 | 164 |
|
49949 | 165 |
lemma mlex_eq [code]: |
166 |
"f <*mlex*> R = {(x, y). f x < f y \<or> (f x \<le> f y \<and> (x, y) \<in> R)}" |
|
167 |
by (auto simp add: mlex_prod_def) |
|
168 |
||
169 |
lemma [code]: |
|
170 |
fixes xs :: "('a::finite \<times> 'a) list" |
|
171 |
shows "acc (set xs) = bacc (set xs) (card_UNIV TYPE('a))" |
|
172 |
by (simp add: card_UNIV_def acc_bacc_eq) |
|
173 |
||
174 |
lemma [code]: |
|
175 |
"accp r = (\<lambda>x. x \<in> acc {(x, y). r x y})" |
|
176 |
by (simp add: acc_def) |
|
40652 | 177 |
|
26348 | 178 |
|
49949 | 179 |
subsection {* Default instances for @{class enum} *} |
26348 | 180 |
|
26444 | 181 |
lemma map_of_zip_enum_is_Some: |
182 |
assumes "length ys = length (enum \<Colon> 'a\<Colon>enum list)" |
|
183 |
shows "\<exists>y. map_of (zip (enum \<Colon> 'a\<Colon>enum list) ys) x = Some y" |
|
184 |
proof - |
|
185 |
from assms have "x \<in> set (enum \<Colon> 'a\<Colon>enum list) \<longleftrightarrow> |
|
186 |
(\<exists>y. map_of (zip (enum \<Colon> 'a\<Colon>enum list) ys) x = Some y)" |
|
187 |
by (auto intro!: map_of_zip_is_Some) |
|
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
188 |
then show ?thesis using enum_UNIV by auto |
26444 | 189 |
qed |
190 |
||
191 |
lemma map_of_zip_enum_inject: |
|
192 |
fixes xs ys :: "'b\<Colon>enum list" |
|
193 |
assumes length: "length xs = length (enum \<Colon> 'a\<Colon>enum list)" |
|
194 |
"length ys = length (enum \<Colon> 'a\<Colon>enum list)" |
|
195 |
and map_of: "the \<circ> map_of (zip (enum \<Colon> 'a\<Colon>enum list) xs) = the \<circ> map_of (zip (enum \<Colon> 'a\<Colon>enum list) ys)" |
|
196 |
shows "xs = ys" |
|
197 |
proof - |
|
198 |
have "map_of (zip (enum \<Colon> 'a list) xs) = map_of (zip (enum \<Colon> 'a list) ys)" |
|
199 |
proof |
|
200 |
fix x :: 'a |
|
201 |
from length map_of_zip_enum_is_Some obtain y1 y2 |
|
202 |
where "map_of (zip (enum \<Colon> 'a list) xs) x = Some y1" |
|
203 |
and "map_of (zip (enum \<Colon> 'a list) ys) x = Some y2" by blast |
|
47230 | 204 |
moreover from map_of |
205 |
have "the (map_of (zip (enum \<Colon> 'a\<Colon>enum list) xs) x) = the (map_of (zip (enum \<Colon> 'a\<Colon>enum list) ys) x)" |
|
26444 | 206 |
by (auto dest: fun_cong) |
207 |
ultimately show "map_of (zip (enum \<Colon> 'a\<Colon>enum list) xs) x = map_of (zip (enum \<Colon> 'a\<Colon>enum list) ys) x" |
|
208 |
by simp |
|
209 |
qed |
|
210 |
with length enum_distinct show "xs = ys" by (rule map_of_zip_inject) |
|
211 |
qed |
|
212 |
||
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
213 |
definition all_n_lists :: "(('a :: enum) list \<Rightarrow> bool) \<Rightarrow> nat \<Rightarrow> bool" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
214 |
where |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
215 |
"all_n_lists P n \<longleftrightarrow> (\<forall>xs \<in> set (List.n_lists n enum). P xs)" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
216 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
217 |
lemma [code]: |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
218 |
"all_n_lists P n \<longleftrightarrow> (if n = 0 then P [] else enum_all (%x. all_n_lists (%xs. P (x # xs)) (n - 1)))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
219 |
unfolding all_n_lists_def enum_all |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
220 |
by (cases n) (auto simp add: enum_UNIV) |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
221 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
222 |
definition ex_n_lists :: "(('a :: enum) list \<Rightarrow> bool) \<Rightarrow> nat \<Rightarrow> bool" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
223 |
where |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
224 |
"ex_n_lists P n \<longleftrightarrow> (\<exists>xs \<in> set (List.n_lists n enum). P xs)" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
225 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
226 |
lemma [code]: |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
227 |
"ex_n_lists P n \<longleftrightarrow> (if n = 0 then P [] else enum_ex (%x. ex_n_lists (%xs. P (x # xs)) (n - 1)))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
228 |
unfolding ex_n_lists_def enum_ex |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
229 |
by (cases n) (auto simp add: enum_UNIV) |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
230 |
|
26444 | 231 |
instantiation "fun" :: (enum, enum) enum |
232 |
begin |
|
233 |
||
234 |
definition |
|
49948
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
48123
diff
changeset
|
235 |
"enum = map (\<lambda>ys. the o map_of (zip (enum\<Colon>'a list) ys)) (List.n_lists (length (enum\<Colon>'a\<Colon>enum list)) enum)" |
26444 | 236 |
|
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
237 |
definition |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
238 |
"enum_all P = all_n_lists (\<lambda>bs. P (the o map_of (zip enum bs))) (length (enum :: 'a list))" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
239 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
240 |
definition |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
241 |
"enum_ex P = ex_n_lists (\<lambda>bs. P (the o map_of (zip enum bs))) (length (enum :: 'a list))" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
242 |
|
26444 | 243 |
instance proof |
244 |
show "UNIV = set (enum \<Colon> ('a \<Rightarrow> 'b) list)" |
|
245 |
proof (rule UNIV_eq_I) |
|
246 |
fix f :: "'a \<Rightarrow> 'b" |
|
247 |
have "f = the \<circ> map_of (zip (enum \<Colon> 'a\<Colon>enum list) (map f enum))" |
|
40683 | 248 |
by (auto simp add: map_of_zip_map fun_eq_iff intro: in_enum) |
26444 | 249 |
then show "f \<in> set enum" |
40683 | 250 |
by (auto simp add: enum_fun_def set_n_lists intro: in_enum) |
26444 | 251 |
qed |
252 |
next |
|
253 |
from map_of_zip_enum_inject |
|
254 |
show "distinct (enum \<Colon> ('a \<Rightarrow> 'b) list)" |
|
255 |
by (auto intro!: inj_onI simp add: enum_fun_def |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
256 |
distinct_map distinct_n_lists enum_distinct set_n_lists) |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
257 |
next |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
258 |
fix P |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
259 |
show "enum_all (P :: ('a \<Rightarrow> 'b) \<Rightarrow> bool) = Ball UNIV P" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
260 |
proof |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
261 |
assume "enum_all P" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
262 |
show "Ball UNIV P" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
263 |
proof |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
264 |
fix f :: "'a \<Rightarrow> 'b" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
265 |
have f: "f = the \<circ> map_of (zip (enum \<Colon> 'a\<Colon>enum list) (map f enum))" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
266 |
by (auto simp add: map_of_zip_map fun_eq_iff intro: in_enum) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
267 |
from `enum_all P` have "P (the \<circ> map_of (zip enum (map f enum)))" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
268 |
unfolding enum_all_fun_def all_n_lists_def |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
269 |
apply (simp add: set_n_lists) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
270 |
apply (erule_tac x="map f enum" in allE) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
271 |
apply (auto intro!: in_enum) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
272 |
done |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
273 |
from this f show "P f" by auto |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
274 |
qed |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
275 |
next |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
276 |
assume "Ball UNIV P" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
277 |
from this show "enum_all P" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
278 |
unfolding enum_all_fun_def all_n_lists_def by auto |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
279 |
qed |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
280 |
next |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
281 |
fix P |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
282 |
show "enum_ex (P :: ('a \<Rightarrow> 'b) \<Rightarrow> bool) = Bex UNIV P" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
283 |
proof |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
284 |
assume "enum_ex P" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
285 |
from this show "Bex UNIV P" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
286 |
unfolding enum_ex_fun_def ex_n_lists_def by auto |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
287 |
next |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
288 |
assume "Bex UNIV P" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
289 |
from this obtain f where "P f" .. |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
290 |
have f: "f = the \<circ> map_of (zip (enum \<Colon> 'a\<Colon>enum list) (map f enum))" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
291 |
by (auto simp add: map_of_zip_map fun_eq_iff intro: in_enum) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
292 |
from `P f` this have "P (the \<circ> map_of (zip (enum \<Colon> 'a\<Colon>enum list) (map f enum)))" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
293 |
by auto |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
294 |
from this show "enum_ex P" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
295 |
unfolding enum_ex_fun_def ex_n_lists_def |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
296 |
apply (auto simp add: set_n_lists) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
297 |
apply (rule_tac x="map f enum" in exI) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
298 |
apply (auto intro!: in_enum) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
299 |
done |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
300 |
qed |
26444 | 301 |
qed |
302 |
||
303 |
end |
|
304 |
||
38857
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
haftmann
parents:
37765
diff
changeset
|
305 |
lemma enum_fun_code [code]: "enum = (let enum_a = (enum \<Colon> 'a\<Colon>{enum, equal} list) |
49948
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
48123
diff
changeset
|
306 |
in map (\<lambda>ys. the o map_of (zip enum_a ys)) (List.n_lists (length enum_a) enum))" |
28245
9767dd8e1e54
celver code lemma avoid type ambiguity problem with Haskell
haftmann
parents:
27487
diff
changeset
|
307 |
by (simp add: enum_fun_def Let_def) |
26444 | 308 |
|
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
309 |
lemma enum_all_fun_code [code]: |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
310 |
"enum_all P = (let enum_a = (enum :: 'a::{enum, equal} list) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
311 |
in all_n_lists (\<lambda>bs. P (the o map_of (zip enum_a bs))) (length enum_a))" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
312 |
by (simp only: enum_all_fun_def Let_def) |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
313 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
314 |
lemma enum_ex_fun_code [code]: |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
315 |
"enum_ex P = (let enum_a = (enum :: 'a::{enum, equal} list) |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
316 |
in ex_n_lists (\<lambda>bs. P (the o map_of (zip enum_a bs))) (length enum_a))" |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
317 |
by (simp only: enum_ex_fun_def Let_def) |
45963
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
318 |
|
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
319 |
instantiation set :: (enum) enum |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
320 |
begin |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
321 |
|
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
322 |
definition |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
323 |
"enum = map set (sublists enum)" |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
324 |
|
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
325 |
definition |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
326 |
"enum_all P \<longleftrightarrow> (\<forall>A\<in>set enum. P (A::'a set))" |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
327 |
|
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
328 |
definition |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
329 |
"enum_ex P \<longleftrightarrow> (\<exists>A\<in>set enum. P (A::'a set))" |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
330 |
|
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
331 |
instance proof |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
332 |
qed (simp_all add: enum_set_def enum_all_set_def enum_ex_set_def sublists_powset distinct_set_sublists |
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
333 |
enum_distinct enum_UNIV) |
29024 | 334 |
|
335 |
end |
|
336 |
||
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
337 |
instantiation unit :: enum |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
338 |
begin |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
339 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
340 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
341 |
"enum = [()]" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
342 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
343 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
344 |
"enum_all P = P ()" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
345 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
346 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
347 |
"enum_ex P = P ()" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
348 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
349 |
instance proof |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
350 |
qed (auto simp add: enum_unit_def enum_all_unit_def enum_ex_unit_def) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
351 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
352 |
end |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
353 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
354 |
instantiation bool :: enum |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
355 |
begin |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
356 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
357 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
358 |
"enum = [False, True]" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
359 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
360 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
361 |
"enum_all P \<longleftrightarrow> P False \<and> P True" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
362 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
363 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
364 |
"enum_ex P \<longleftrightarrow> P False \<or> P True" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
365 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
366 |
instance proof |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
367 |
qed (simp_all only: enum_bool_def enum_all_bool_def enum_ex_bool_def UNIV_bool, simp_all) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
368 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
369 |
end |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
370 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
371 |
instantiation prod :: (enum, enum) enum |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
372 |
begin |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
373 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
374 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
375 |
"enum = List.product enum enum" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
376 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
377 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
378 |
"enum_all P = enum_all (%x. enum_all (%y. P (x, y)))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
379 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
380 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
381 |
"enum_ex P = enum_ex (%x. enum_ex (%y. P (x, y)))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
382 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
383 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
384 |
instance by default |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
385 |
(simp_all add: enum_prod_def product_list_set distinct_product |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
386 |
enum_UNIV enum_distinct enum_all_prod_def enum_ex_prod_def) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
387 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
388 |
end |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
389 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
390 |
instantiation sum :: (enum, enum) enum |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
391 |
begin |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
392 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
393 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
394 |
"enum = map Inl enum @ map Inr enum" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
395 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
396 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
397 |
"enum_all P \<longleftrightarrow> enum_all (\<lambda>x. P (Inl x)) \<and> enum_all (\<lambda>x. P (Inr x))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
398 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
399 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
400 |
"enum_ex P \<longleftrightarrow> enum_ex (\<lambda>x. P (Inl x)) \<or> enum_ex (\<lambda>x. P (Inr x))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
401 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
402 |
instance proof |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
403 |
qed (simp_all only: enum_sum_def enum_all_sum_def enum_ex_sum_def UNIV_sum, |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
404 |
auto simp add: enum_UNIV distinct_map enum_distinct) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
405 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
406 |
end |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
407 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
408 |
instantiation nibble :: enum |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
409 |
begin |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
410 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
411 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
412 |
"enum = [Nibble0, Nibble1, Nibble2, Nibble3, Nibble4, Nibble5, Nibble6, Nibble7, |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
413 |
Nibble8, Nibble9, NibbleA, NibbleB, NibbleC, NibbleD, NibbleE, NibbleF]" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
414 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
415 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
416 |
"enum_all P \<longleftrightarrow> P Nibble0 \<and> P Nibble1 \<and> P Nibble2 \<and> P Nibble3 \<and> P Nibble4 \<and> P Nibble5 \<and> P Nibble6 \<and> P Nibble7 |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
417 |
\<and> P Nibble8 \<and> P Nibble9 \<and> P NibbleA \<and> P NibbleB \<and> P NibbleC \<and> P NibbleD \<and> P NibbleE \<and> P NibbleF" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
418 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
419 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
420 |
"enum_ex P \<longleftrightarrow> P Nibble0 \<or> P Nibble1 \<or> P Nibble2 \<or> P Nibble3 \<or> P Nibble4 \<or> P Nibble5 \<or> P Nibble6 \<or> P Nibble7 |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
421 |
\<or> P Nibble8 \<or> P Nibble9 \<or> P NibbleA \<or> P NibbleB \<or> P NibbleC \<or> P NibbleD \<or> P NibbleE \<or> P NibbleF" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
422 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
423 |
instance proof |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
424 |
qed (simp_all only: enum_nibble_def enum_all_nibble_def enum_ex_nibble_def UNIV_nibble, simp_all) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
425 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
426 |
end |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
427 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
428 |
instantiation char :: enum |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
429 |
begin |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
430 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
431 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
432 |
"enum = chars" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
433 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
434 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
435 |
"enum_all P \<longleftrightarrow> list_all P chars" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
436 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
437 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
438 |
"enum_ex P \<longleftrightarrow> list_ex P chars" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
439 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
440 |
instance proof |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
441 |
qed (simp_all only: enum_char_def enum_all_char_def enum_ex_char_def UNIV_set_chars distinct_chars, |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
442 |
simp_all add: list_all_iff list_ex_iff) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
443 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
444 |
end |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
445 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
446 |
instantiation option :: (enum) enum |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
447 |
begin |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
448 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
449 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
450 |
"enum = None # map Some enum" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
451 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
452 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
453 |
"enum_all P \<longleftrightarrow> P None \<and> enum_all (\<lambda>x. P (Some x))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
454 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
455 |
definition |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
456 |
"enum_ex P \<longleftrightarrow> P None \<or> enum_ex (\<lambda>x. P (Some x))" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
457 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
458 |
instance proof |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
459 |
qed (simp_all only: enum_option_def enum_all_option_def enum_ex_option_def UNIV_option_conv, |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
460 |
auto simp add: distinct_map enum_UNIV enum_distinct) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
461 |
|
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
462 |
end |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
463 |
|
45963
1c7e6454883e
enum type class instance for `set`; dropped misfitting code lemma for trancl
haftmann
parents:
45144
diff
changeset
|
464 |
|
40647 | 465 |
subsection {* Small finite types *} |
466 |
||
467 |
text {* We define small finite types for the use in Quickcheck *} |
|
468 |
||
469 |
datatype finite_1 = a\<^isub>1 |
|
470 |
||
40900
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
471 |
notation (output) a\<^isub>1 ("a\<^isub>1") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
472 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
473 |
lemma UNIV_finite_1: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
474 |
"UNIV = {a\<^isub>1}" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
475 |
by (auto intro: finite_1.exhaust) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
476 |
|
40647 | 477 |
instantiation finite_1 :: enum |
478 |
begin |
|
479 |
||
480 |
definition |
|
481 |
"enum = [a\<^isub>1]" |
|
482 |
||
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
483 |
definition |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
484 |
"enum_all P = P a\<^isub>1" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
485 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
486 |
definition |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
487 |
"enum_ex P = P a\<^isub>1" |
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
488 |
|
40647 | 489 |
instance proof |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
490 |
qed (simp_all only: enum_finite_1_def enum_all_finite_1_def enum_ex_finite_1_def UNIV_finite_1, simp_all) |
40647 | 491 |
|
29024 | 492 |
end |
40647 | 493 |
|
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
494 |
instantiation finite_1 :: linorder |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
495 |
begin |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
496 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
497 |
definition less_finite_1 :: "finite_1 \<Rightarrow> finite_1 \<Rightarrow> bool" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
498 |
where |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
499 |
"x < (y :: finite_1) \<longleftrightarrow> False" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
500 |
|
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
501 |
definition less_eq_finite_1 :: "finite_1 \<Rightarrow> finite_1 \<Rightarrow> bool" |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
502 |
where |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
503 |
"x \<le> (y :: finite_1) \<longleftrightarrow> True" |
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
504 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
505 |
instance |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
506 |
apply (intro_classes) |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
507 |
apply (auto simp add: less_finite_1_def less_eq_finite_1_def) |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
508 |
apply (metis finite_1.exhaust) |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
509 |
done |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
510 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
511 |
end |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
512 |
|
41085
a549ff1d4070
adding a smarter enumeration scheme for finite functions
bulwahn
parents:
41078
diff
changeset
|
513 |
hide_const (open) a\<^isub>1 |
40657 | 514 |
|
40647 | 515 |
datatype finite_2 = a\<^isub>1 | a\<^isub>2 |
516 |
||
40900
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
517 |
notation (output) a\<^isub>1 ("a\<^isub>1") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
518 |
notation (output) a\<^isub>2 ("a\<^isub>2") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
519 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
520 |
lemma UNIV_finite_2: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
521 |
"UNIV = {a\<^isub>1, a\<^isub>2}" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
522 |
by (auto intro: finite_2.exhaust) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
523 |
|
40647 | 524 |
instantiation finite_2 :: enum |
525 |
begin |
|
526 |
||
527 |
definition |
|
528 |
"enum = [a\<^isub>1, a\<^isub>2]" |
|
529 |
||
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
530 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
531 |
"enum_all P \<longleftrightarrow> P a\<^isub>1 \<and> P a\<^isub>2" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
532 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
533 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
534 |
"enum_ex P \<longleftrightarrow> P a\<^isub>1 \<or> P a\<^isub>2" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
535 |
|
40647 | 536 |
instance proof |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
537 |
qed (simp_all only: enum_finite_2_def enum_all_finite_2_def enum_ex_finite_2_def UNIV_finite_2, simp_all) |
40647 | 538 |
|
539 |
end |
|
540 |
||
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
541 |
instantiation finite_2 :: linorder |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
542 |
begin |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
543 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
544 |
definition less_finite_2 :: "finite_2 \<Rightarrow> finite_2 \<Rightarrow> bool" |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
545 |
where |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
546 |
"x < y \<longleftrightarrow> x = a\<^isub>1 \<and> y = a\<^isub>2" |
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
547 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
548 |
definition less_eq_finite_2 :: "finite_2 \<Rightarrow> finite_2 \<Rightarrow> bool" |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
549 |
where |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
550 |
"x \<le> y \<longleftrightarrow> x = y \<or> x < (y :: finite_2)" |
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
551 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
552 |
instance |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
553 |
apply (intro_classes) |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
554 |
apply (auto simp add: less_finite_2_def less_eq_finite_2_def) |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
555 |
apply (metis finite_2.nchotomy)+ |
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
556 |
done |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
557 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
558 |
end |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
559 |
|
41085
a549ff1d4070
adding a smarter enumeration scheme for finite functions
bulwahn
parents:
41078
diff
changeset
|
560 |
hide_const (open) a\<^isub>1 a\<^isub>2 |
40657 | 561 |
|
40647 | 562 |
datatype finite_3 = a\<^isub>1 | a\<^isub>2 | a\<^isub>3 |
563 |
||
40900
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
564 |
notation (output) a\<^isub>1 ("a\<^isub>1") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
565 |
notation (output) a\<^isub>2 ("a\<^isub>2") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
566 |
notation (output) a\<^isub>3 ("a\<^isub>3") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
567 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
568 |
lemma UNIV_finite_3: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
569 |
"UNIV = {a\<^isub>1, a\<^isub>2, a\<^isub>3}" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
570 |
by (auto intro: finite_3.exhaust) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
571 |
|
40647 | 572 |
instantiation finite_3 :: enum |
573 |
begin |
|
574 |
||
575 |
definition |
|
576 |
"enum = [a\<^isub>1, a\<^isub>2, a\<^isub>3]" |
|
577 |
||
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
578 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
579 |
"enum_all P \<longleftrightarrow> P a\<^isub>1 \<and> P a\<^isub>2 \<and> P a\<^isub>3" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
580 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
581 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
582 |
"enum_ex P \<longleftrightarrow> P a\<^isub>1 \<or> P a\<^isub>2 \<or> P a\<^isub>3" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
583 |
|
40647 | 584 |
instance proof |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
585 |
qed (simp_all only: enum_finite_3_def enum_all_finite_3_def enum_ex_finite_3_def UNIV_finite_3, simp_all) |
40647 | 586 |
|
587 |
end |
|
588 |
||
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
589 |
instantiation finite_3 :: linorder |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
590 |
begin |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
591 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
592 |
definition less_finite_3 :: "finite_3 \<Rightarrow> finite_3 \<Rightarrow> bool" |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
593 |
where |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
594 |
"x < y = (case x of a\<^isub>1 \<Rightarrow> y \<noteq> a\<^isub>1 | a\<^isub>2 \<Rightarrow> y = a\<^isub>3 | a\<^isub>3 \<Rightarrow> False)" |
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
595 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
596 |
definition less_eq_finite_3 :: "finite_3 \<Rightarrow> finite_3 \<Rightarrow> bool" |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
597 |
where |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
598 |
"x \<le> y \<longleftrightarrow> x = y \<or> x < (y :: finite_3)" |
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
599 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
600 |
instance proof (intro_classes) |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
601 |
qed (auto simp add: less_finite_3_def less_eq_finite_3_def split: finite_3.split_asm) |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
602 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
603 |
end |
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
604 |
|
41085
a549ff1d4070
adding a smarter enumeration scheme for finite functions
bulwahn
parents:
41078
diff
changeset
|
605 |
hide_const (open) a\<^isub>1 a\<^isub>2 a\<^isub>3 |
40657 | 606 |
|
40647 | 607 |
datatype finite_4 = a\<^isub>1 | a\<^isub>2 | a\<^isub>3 | a\<^isub>4 |
608 |
||
40900
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
609 |
notation (output) a\<^isub>1 ("a\<^isub>1") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
610 |
notation (output) a\<^isub>2 ("a\<^isub>2") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
611 |
notation (output) a\<^isub>3 ("a\<^isub>3") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
612 |
notation (output) a\<^isub>4 ("a\<^isub>4") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
613 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
614 |
lemma UNIV_finite_4: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
615 |
"UNIV = {a\<^isub>1, a\<^isub>2, a\<^isub>3, a\<^isub>4}" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
616 |
by (auto intro: finite_4.exhaust) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
617 |
|
40647 | 618 |
instantiation finite_4 :: enum |
619 |
begin |
|
620 |
||
621 |
definition |
|
622 |
"enum = [a\<^isub>1, a\<^isub>2, a\<^isub>3, a\<^isub>4]" |
|
623 |
||
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
624 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
625 |
"enum_all P \<longleftrightarrow> P a\<^isub>1 \<and> P a\<^isub>2 \<and> P a\<^isub>3 \<and> P a\<^isub>4" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
626 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
627 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
628 |
"enum_ex P \<longleftrightarrow> P a\<^isub>1 \<or> P a\<^isub>2 \<or> P a\<^isub>3 \<or> P a\<^isub>4" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
629 |
|
40647 | 630 |
instance proof |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
631 |
qed (simp_all only: enum_finite_4_def enum_all_finite_4_def enum_ex_finite_4_def UNIV_finite_4, simp_all) |
40647 | 632 |
|
633 |
end |
|
634 |
||
41085
a549ff1d4070
adding a smarter enumeration scheme for finite functions
bulwahn
parents:
41078
diff
changeset
|
635 |
hide_const (open) a\<^isub>1 a\<^isub>2 a\<^isub>3 a\<^isub>4 |
40651
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
636 |
|
9752ba7348b5
adding code equation for function equality; adding some instantiations for the finite types
bulwahn
parents:
40650
diff
changeset
|
637 |
|
40647 | 638 |
datatype finite_5 = a\<^isub>1 | a\<^isub>2 | a\<^isub>3 | a\<^isub>4 | a\<^isub>5 |
639 |
||
40900
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
640 |
notation (output) a\<^isub>1 ("a\<^isub>1") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
641 |
notation (output) a\<^isub>2 ("a\<^isub>2") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
642 |
notation (output) a\<^isub>3 ("a\<^isub>3") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
643 |
notation (output) a\<^isub>4 ("a\<^isub>4") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
644 |
notation (output) a\<^isub>5 ("a\<^isub>5") |
1d5f76d79856
adding shorter output syntax for the finite types of quickcheck
bulwahn
parents:
40898
diff
changeset
|
645 |
|
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
646 |
lemma UNIV_finite_5: |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
647 |
"UNIV = {a\<^isub>1, a\<^isub>2, a\<^isub>3, a\<^isub>4, a\<^isub>5}" |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
648 |
by (auto intro: finite_5.exhaust) |
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
649 |
|
40647 | 650 |
instantiation finite_5 :: enum |
651 |
begin |
|
652 |
||
653 |
definition |
|
654 |
"enum = [a\<^isub>1, a\<^isub>2, a\<^isub>3, a\<^isub>4, a\<^isub>5]" |
|
655 |
||
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
656 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
657 |
"enum_all P \<longleftrightarrow> P a\<^isub>1 \<and> P a\<^isub>2 \<and> P a\<^isub>3 \<and> P a\<^isub>4 \<and> P a\<^isub>5" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
658 |
|
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
659 |
definition |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
660 |
"enum_ex P \<longleftrightarrow> P a\<^isub>1 \<or> P a\<^isub>2 \<or> P a\<^isub>3 \<or> P a\<^isub>4 \<or> P a\<^isub>5" |
41078
051251fde456
adding more efficient implementations for quantifiers in Enum
bulwahn
parents:
40900
diff
changeset
|
661 |
|
40647 | 662 |
instance proof |
49950
cd882d53ba6b
tailored enum specification towards simple instantiation;
haftmann
parents:
49949
diff
changeset
|
663 |
qed (simp_all only: enum_finite_5_def enum_all_finite_5_def enum_ex_finite_5_def UNIV_finite_5, simp_all) |
40647 | 664 |
|
665 |
end |
|
666 |
||
46352
73b03235799a
an executable version of accessible part (only for finite types yet)
bulwahn
parents:
46336
diff
changeset
|
667 |
hide_const (open) a\<^isub>1 a\<^isub>2 a\<^isub>3 a\<^isub>4 a\<^isub>5 |
73b03235799a
an executable version of accessible part (only for finite types yet)
bulwahn
parents:
46336
diff
changeset
|
668 |
|
49948
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
48123
diff
changeset
|
669 |
|
46352
73b03235799a
an executable version of accessible part (only for finite types yet)
bulwahn
parents:
46336
diff
changeset
|
670 |
subsection {* Closing up *} |
40657 | 671 |
|
41085
a549ff1d4070
adding a smarter enumeration scheme for finite functions
bulwahn
parents:
41078
diff
changeset
|
672 |
hide_type (open) finite_1 finite_2 finite_3 finite_4 finite_5 |
49948
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
48123
diff
changeset
|
673 |
hide_const (open) enum enum_all enum_ex all_n_lists ex_n_lists ntrancl |
40647 | 674 |
|
675 |
end |
|
49948
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
48123
diff
changeset
|
676 |