author | wenzelm |
Fri, 18 Mar 2016 17:58:19 +0100 | |
changeset 62668 | 360d3464919c |
parent 62597 | b3f2b8c906a6 |
child 67091 | 1393c2340eec |
permissions | -rw-r--r-- |
37653 | 1 |
(* Title: HOL/Library/Cardinality.thy |
48051 | 2 |
Author: Brian Huffman, Andreas Lochbihler |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
3 |
*) |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
4 |
|
60500 | 5 |
section \<open>Cardinality of types\<close> |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
6 |
|
37653 | 7 |
theory Cardinality |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
8 |
imports Phantom_Type |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
9 |
begin |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
10 |
|
60500 | 11 |
subsection \<open>Preliminary lemmas\<close> |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
12 |
(* These should be moved elsewhere *) |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
13 |
|
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
14 |
lemma (in type_definition) univ: |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
15 |
"UNIV = Abs ` A" |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
16 |
proof |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
17 |
show "Abs ` A \<subseteq> UNIV" by (rule subset_UNIV) |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
18 |
show "UNIV \<subseteq> Abs ` A" |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
19 |
proof |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
20 |
fix x :: 'b |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
21 |
have "x = Abs (Rep x)" by (rule Rep_inverse [symmetric]) |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
22 |
moreover have "Rep x \<in> A" by (rule Rep) |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
23 |
ultimately show "x \<in> Abs ` A" by (rule image_eqI) |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
24 |
qed |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
25 |
qed |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
26 |
|
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
27 |
lemma (in type_definition) card: "card (UNIV :: 'b set) = card A" |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
28 |
by (simp add: univ card_image inj_on_def Abs_inject) |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
29 |
|
48060 | 30 |
lemma finite_range_Some: "finite (range (Some :: 'a \<Rightarrow> 'a option)) = finite (UNIV :: 'a set)" |
31 |
by(auto dest: finite_imageD intro: inj_Some) |
|
32 |
||
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
33 |
lemma infinite_literal: "\<not> finite (UNIV :: String.literal set)" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
34 |
proof - |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
35 |
have "inj STR" by(auto intro: injI) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
36 |
thus ?thesis |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
37 |
by(auto simp add: type_definition.univ[OF type_definition_literal] infinite_UNIV_listI dest: finite_imageD) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
38 |
qed |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
39 |
|
60500 | 40 |
subsection \<open>Cardinalities of types\<close> |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
41 |
|
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
42 |
syntax "_type_card" :: "type => nat" ("(1CARD/(1'(_')))") |
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
43 |
|
61076 | 44 |
translations "CARD('t)" => "CONST card (CONST UNIV :: 't set)" |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
45 |
|
60500 | 46 |
print_translation \<open> |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
47 |
let |
52147 | 48 |
fun card_univ_tr' ctxt [Const (@{const_syntax UNIV}, Type (_, [T]))] = |
49689
b8a710806de9
recovered print translation after 'a => bool to 'a set change;
wenzelm
parents:
48176
diff
changeset
|
49 |
Syntax.const @{syntax_const "_type_card"} $ Syntax_Phases.term_of_typ ctxt T |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
50 |
in [(@{const_syntax card}, card_univ_tr')] end |
60500 | 51 |
\<close> |
24407 | 52 |
|
48058 | 53 |
lemma card_prod [simp]: "CARD('a \<times> 'b) = CARD('a) * CARD('b)" |
26153 | 54 |
unfolding UNIV_Times_UNIV [symmetric] by (simp only: card_cartesian_product) |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
55 |
|
48060 | 56 |
lemma card_UNIV_sum: "CARD('a + 'b) = (if CARD('a) \<noteq> 0 \<and> CARD('b) \<noteq> 0 then CARD('a) + CARD('b) else 0)" |
57 |
unfolding UNIV_Plus_UNIV[symmetric] |
|
58 |
by(auto simp add: card_eq_0_iff card_Plus simp del: UNIV_Plus_UNIV) |
|
59 |
||
30001 | 60 |
lemma card_sum [simp]: "CARD('a + 'b) = CARD('a::finite) + CARD('b::finite)" |
48060 | 61 |
by(simp add: card_UNIV_sum) |
62 |
||
63 |
lemma card_UNIV_option: "CARD('a option) = (if CARD('a) = 0 then 0 else CARD('a) + 1)" |
|
64 |
proof - |
|
65 |
have "(None :: 'a option) \<notin> range Some" by clarsimp |
|
66 |
thus ?thesis |
|
53191 | 67 |
by (simp add: UNIV_option_conv card_eq_0_iff finite_range_Some card_image) |
48060 | 68 |
qed |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
69 |
|
30001 | 70 |
lemma card_option [simp]: "CARD('a option) = Suc CARD('a::finite)" |
48060 | 71 |
by(simp add: card_UNIV_option) |
72 |
||
73 |
lemma card_UNIV_set: "CARD('a set) = (if CARD('a) = 0 then 0 else 2 ^ CARD('a))" |
|
74 |
by(simp add: Pow_UNIV[symmetric] card_eq_0_iff card_Pow del: Pow_UNIV) |
|
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
75 |
|
30001 | 76 |
lemma card_set [simp]: "CARD('a set) = 2 ^ CARD('a::finite)" |
48060 | 77 |
by(simp add: card_UNIV_set) |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
diff
changeset
|
78 |
|
30001 | 79 |
lemma card_nat [simp]: "CARD(nat) = 0" |
44142 | 80 |
by (simp add: card_eq_0_iff) |
30001 | 81 |
|
48060 | 82 |
lemma card_fun: "CARD('a \<Rightarrow> 'b) = (if CARD('a) \<noteq> 0 \<and> CARD('b) \<noteq> 0 \<or> CARD('b) = 1 then CARD('b) ^ CARD('a) else 0)" |
83 |
proof - |
|
84 |
{ assume "0 < CARD('a)" and "0 < CARD('b)" |
|
85 |
hence fina: "finite (UNIV :: 'a set)" and finb: "finite (UNIV :: 'b set)" |
|
86 |
by(simp_all only: card_ge_0_finite) |
|
87 |
from finite_distinct_list[OF finb] obtain bs |
|
88 |
where bs: "set bs = (UNIV :: 'b set)" and distb: "distinct bs" by blast |
|
89 |
from finite_distinct_list[OF fina] obtain as |
|
90 |
where as: "set as = (UNIV :: 'a set)" and dista: "distinct as" by blast |
|
91 |
have cb: "CARD('b) = length bs" |
|
92 |
unfolding bs[symmetric] distinct_card[OF distb] .. |
|
93 |
have ca: "CARD('a) = length as" |
|
94 |
unfolding as[symmetric] distinct_card[OF dista] .. |
|
49948
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
49689
diff
changeset
|
95 |
let ?xs = "map (\<lambda>ys. the o map_of (zip as ys)) (List.n_lists (length as) bs)" |
48060 | 96 |
have "UNIV = set ?xs" |
97 |
proof(rule UNIV_eq_I) |
|
98 |
fix f :: "'a \<Rightarrow> 'b" |
|
99 |
from as have "f = the \<circ> map_of (zip as (map f as))" |
|
100 |
by(auto simp add: map_of_zip_map) |
|
101 |
thus "f \<in> set ?xs" using bs by(auto simp add: set_n_lists) |
|
102 |
qed |
|
103 |
moreover have "distinct ?xs" unfolding distinct_map |
|
104 |
proof(intro conjI distinct_n_lists distb inj_onI) |
|
105 |
fix xs ys :: "'b list" |
|
49948
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
49689
diff
changeset
|
106 |
assume xs: "xs \<in> set (List.n_lists (length as) bs)" |
744934b818c7
moved quite generic material from theory Enum to more appropriate places
haftmann
parents:
49689
diff
changeset
|
107 |
and ys: "ys \<in> set (List.n_lists (length as) bs)" |
48060 | 108 |
and eq: "the \<circ> map_of (zip as xs) = the \<circ> map_of (zip as ys)" |
109 |
from xs ys have [simp]: "length xs = length as" "length ys = length as" |
|
110 |
by(simp_all add: length_n_lists_elem) |
|
111 |
have "map_of (zip as xs) = map_of (zip as ys)" |
|
112 |
proof |
|
113 |
fix x |
|
114 |
from as bs have "\<exists>y. map_of (zip as xs) x = Some y" "\<exists>y. map_of (zip as ys) x = Some y" |
|
115 |
by(simp_all add: map_of_zip_is_Some[symmetric]) |
|
116 |
with eq show "map_of (zip as xs) x = map_of (zip as ys) x" |
|
117 |
by(auto dest: fun_cong[where x=x]) |
|
118 |
qed |
|
119 |
with dista show "xs = ys" by(simp add: map_of_zip_inject) |
|
120 |
qed |
|
121 |
hence "card (set ?xs) = length ?xs" by(simp only: distinct_card) |
|
122 |
moreover have "length ?xs = length bs ^ length as" by(simp add: length_n_lists) |
|
123 |
ultimately have "CARD('a \<Rightarrow> 'b) = CARD('b) ^ CARD('a)" using cb ca by simp } |
|
124 |
moreover { |
|
125 |
assume cb: "CARD('b) = 1" |
|
126 |
then obtain b where b: "UNIV = {b :: 'b}" by(auto simp add: card_Suc_eq) |
|
127 |
have eq: "UNIV = {\<lambda>x :: 'a. b ::'b}" |
|
128 |
proof(rule UNIV_eq_I) |
|
129 |
fix x :: "'a \<Rightarrow> 'b" |
|
130 |
{ fix y |
|
131 |
have "x y \<in> UNIV" .. |
|
132 |
hence "x y = b" unfolding b by simp } |
|
133 |
thus "x \<in> {\<lambda>x. b}" by(auto) |
|
134 |
qed |
|
135 |
have "CARD('a \<Rightarrow> 'b) = 1" unfolding eq by simp } |
|
136 |
ultimately show ?thesis |
|
137 |
by(auto simp del: One_nat_def)(auto simp add: card_eq_0_iff dest: finite_fun_UNIVD2 finite_fun_UNIVD1) |
|
138 |
qed |
|
139 |
||
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
140 |
corollary finite_UNIV_fun: |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
141 |
"finite (UNIV :: ('a \<Rightarrow> 'b) set) \<longleftrightarrow> |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
142 |
finite (UNIV :: 'a set) \<and> finite (UNIV :: 'b set) \<or> CARD('b) = 1" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
143 |
(is "?lhs \<longleftrightarrow> ?rhs") |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
144 |
proof - |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
145 |
have "?lhs \<longleftrightarrow> CARD('a \<Rightarrow> 'b) > 0" by(simp add: card_gt_0_iff) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
146 |
also have "\<dots> \<longleftrightarrow> CARD('a) > 0 \<and> CARD('b) > 0 \<or> CARD('b) = 1" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
147 |
by(simp add: card_fun) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
148 |
also have "\<dots> = ?rhs" by(simp add: card_gt_0_iff) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
149 |
finally show ?thesis . |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
150 |
qed |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
151 |
|
48060 | 152 |
lemma card_literal: "CARD(String.literal) = 0" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
153 |
by(simp add: card_eq_0_iff infinite_literal) |
30001 | 154 |
|
60500 | 155 |
subsection \<open>Classes with at least 1 and 2\<close> |
30001 | 156 |
|
60500 | 157 |
text \<open>Class finite already captures "at least 1"\<close> |
30001 | 158 |
|
159 |
lemma zero_less_card_finite [simp]: "0 < CARD('a::finite)" |
|
29997 | 160 |
unfolding neq0_conv [symmetric] by simp |
161 |
||
30001 | 162 |
lemma one_le_card_finite [simp]: "Suc 0 \<le> CARD('a::finite)" |
163 |
by (simp add: less_Suc_eq_le [symmetric]) |
|
164 |
||
60500 | 165 |
text \<open>Class for cardinality "at least 2"\<close> |
30001 | 166 |
|
167 |
class card2 = finite + |
|
168 |
assumes two_le_card: "2 \<le> CARD('a)" |
|
169 |
||
170 |
lemma one_less_card: "Suc 0 < CARD('a::card2)" |
|
171 |
using two_le_card [where 'a='a] by simp |
|
172 |
||
173 |
lemma one_less_int_card: "1 < int CARD('a::card2)" |
|
174 |
using one_less_card [where 'a='a] by simp |
|
175 |
||
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
176 |
|
60500 | 177 |
subsection \<open>A type class for deciding finiteness of types\<close> |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
178 |
|
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
179 |
type_synonym 'a finite_UNIV = "('a, bool) phantom" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
180 |
|
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
181 |
class finite_UNIV = |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
182 |
fixes finite_UNIV :: "('a, bool) phantom" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
183 |
assumes finite_UNIV: "finite_UNIV = Phantom('a) (finite (UNIV :: 'a set))" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
184 |
|
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
185 |
lemma finite_UNIV_code [code_unfold]: |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
186 |
"finite (UNIV :: 'a :: finite_UNIV set) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
187 |
\<longleftrightarrow> of_phantom (finite_UNIV :: 'a finite_UNIV)" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
188 |
by(simp add: finite_UNIV) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
189 |
|
60500 | 190 |
subsection \<open>A type class for computing the cardinality of types\<close> |
48051 | 191 |
|
48059 | 192 |
definition is_list_UNIV :: "'a list \<Rightarrow> bool" |
51116
0dac0158b8d4
implement code generation for finite, card, op = and op <= for sets always via finite_UNIV and card_UNIV, as fragile rewrites based on sorts are hard to find and debug
Andreas Lochbihler
parents:
49948
diff
changeset
|
193 |
where "is_list_UNIV xs = (let c = CARD('a) in if c = 0 then False else size (remdups xs) = c)" |
48059 | 194 |
|
195 |
lemma is_list_UNIV_iff: "is_list_UNIV xs \<longleftrightarrow> set xs = UNIV" |
|
196 |
by(auto simp add: is_list_UNIV_def Let_def card_eq_0_iff List.card_set[symmetric] |
|
197 |
dest: subst[where P="finite", OF _ finite_set] card_eq_UNIV_imp_eq_UNIV) |
|
198 |
||
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
199 |
type_synonym 'a card_UNIV = "('a, nat) phantom" |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
200 |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
201 |
class card_UNIV = finite_UNIV + |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
202 |
fixes card_UNIV :: "'a card_UNIV" |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
203 |
assumes card_UNIV: "card_UNIV = Phantom('a) CARD('a)" |
48051 | 204 |
|
61585 | 205 |
subsection \<open>Instantiations for \<open>card_UNIV\<close>\<close> |
48051 | 206 |
|
207 |
instantiation nat :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
208 |
definition "finite_UNIV = Phantom(nat) False" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
209 |
definition "card_UNIV = Phantom(nat) 0" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
210 |
instance by intro_classes (simp_all add: finite_UNIV_nat_def card_UNIV_nat_def) |
48051 | 211 |
end |
212 |
||
213 |
instantiation int :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
214 |
definition "finite_UNIV = Phantom(int) False" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
215 |
definition "card_UNIV = Phantom(int) 0" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
216 |
instance by intro_classes (simp_all add: card_UNIV_int_def finite_UNIV_int_def infinite_UNIV_int) |
48051 | 217 |
end |
218 |
||
51143
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
219 |
instantiation natural :: card_UNIV begin |
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
220 |
definition "finite_UNIV = Phantom(natural) False" |
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
221 |
definition "card_UNIV = Phantom(natural) 0" |
60679 | 222 |
instance |
223 |
by standard |
|
224 |
(auto simp add: finite_UNIV_natural_def card_UNIV_natural_def card_eq_0_iff |
|
225 |
type_definition.univ [OF type_definition_natural] natural_eq_iff |
|
226 |
dest!: finite_imageD intro: inj_onI) |
|
51143
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
227 |
end |
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
228 |
|
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
229 |
instantiation integer :: card_UNIV begin |
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
230 |
definition "finite_UNIV = Phantom(integer) False" |
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
51139
diff
changeset
|
231 |
definition "card_UNIV = Phantom(integer) 0" |
60679 | 232 |
instance |
233 |
by standard |
|
234 |
(auto simp add: finite_UNIV_integer_def card_UNIV_integer_def card_eq_0_iff |
|
235 |
type_definition.univ [OF type_definition_integer] infinite_UNIV_int |
|
236 |
dest!: finite_imageD intro: inj_onI) |
|
48165
d07a0b9601aa
instantiate card_UNIV with nibble and code_numeral
Andreas Lochbihler
parents:
48164
diff
changeset
|
237 |
end |
d07a0b9601aa
instantiate card_UNIV with nibble and code_numeral
Andreas Lochbihler
parents:
48164
diff
changeset
|
238 |
|
48051 | 239 |
instantiation list :: (type) card_UNIV begin |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
240 |
definition "finite_UNIV = Phantom('a list) False" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
241 |
definition "card_UNIV = Phantom('a list) 0" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
242 |
instance by intro_classes (simp_all add: card_UNIV_list_def finite_UNIV_list_def infinite_UNIV_listI) |
48051 | 243 |
end |
244 |
||
245 |
instantiation unit :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
246 |
definition "finite_UNIV = Phantom(unit) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
247 |
definition "card_UNIV = Phantom(unit) 1" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
248 |
instance by intro_classes (simp_all add: card_UNIV_unit_def finite_UNIV_unit_def) |
48051 | 249 |
end |
250 |
||
251 |
instantiation bool :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
252 |
definition "finite_UNIV = Phantom(bool) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
253 |
definition "card_UNIV = Phantom(bool) 2" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
254 |
instance by(intro_classes)(simp_all add: card_UNIV_bool_def finite_UNIV_bool_def) |
48051 | 255 |
end |
256 |
||
257 |
instantiation char :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
258 |
definition "finite_UNIV = Phantom(char) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
259 |
definition "card_UNIV = Phantom(char) 256" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
260 |
instance by intro_classes (simp_all add: card_UNIV_char_def card_UNIV_char finite_UNIV_char_def) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
261 |
end |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
262 |
|
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
263 |
instantiation prod :: (finite_UNIV, finite_UNIV) finite_UNIV begin |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
264 |
definition "finite_UNIV = Phantom('a \<times> 'b) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
265 |
(of_phantom (finite_UNIV :: 'a finite_UNIV) \<and> of_phantom (finite_UNIV :: 'b finite_UNIV))" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
266 |
instance by intro_classes (simp add: finite_UNIV_prod_def finite_UNIV finite_prod) |
48051 | 267 |
end |
268 |
||
269 |
instantiation prod :: (card_UNIV, card_UNIV) card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
270 |
definition "card_UNIV = Phantom('a \<times> 'b) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
271 |
(of_phantom (card_UNIV :: 'a card_UNIV) * of_phantom (card_UNIV :: 'b card_UNIV))" |
48060 | 272 |
instance by intro_classes (simp add: card_UNIV_prod_def card_UNIV) |
48051 | 273 |
end |
274 |
||
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
275 |
instantiation sum :: (finite_UNIV, finite_UNIV) finite_UNIV begin |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
276 |
definition "finite_UNIV = Phantom('a + 'b) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
277 |
(of_phantom (finite_UNIV :: 'a finite_UNIV) \<and> of_phantom (finite_UNIV :: 'b finite_UNIV))" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
278 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
279 |
by intro_classes (simp add: UNIV_Plus_UNIV[symmetric] finite_UNIV_sum_def finite_UNIV del: UNIV_Plus_UNIV) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
280 |
end |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
281 |
|
48051 | 282 |
instantiation sum :: (card_UNIV, card_UNIV) card_UNIV begin |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
283 |
definition "card_UNIV = Phantom('a + 'b) |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
284 |
(let ca = of_phantom (card_UNIV :: 'a card_UNIV); |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
285 |
cb = of_phantom (card_UNIV :: 'b card_UNIV) |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
286 |
in if ca \<noteq> 0 \<and> cb \<noteq> 0 then ca + cb else 0)" |
48060 | 287 |
instance by intro_classes (auto simp add: card_UNIV_sum_def card_UNIV card_UNIV_sum) |
48051 | 288 |
end |
289 |
||
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
290 |
instantiation "fun" :: (finite_UNIV, card_UNIV) finite_UNIV begin |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
291 |
definition "finite_UNIV = Phantom('a \<Rightarrow> 'b) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
292 |
(let cb = of_phantom (card_UNIV :: 'b card_UNIV) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
293 |
in cb = 1 \<or> of_phantom (finite_UNIV :: 'a finite_UNIV) \<and> cb \<noteq> 0)" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
294 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
295 |
by intro_classes (auto simp add: finite_UNIV_fun_def Let_def card_UNIV finite_UNIV finite_UNIV_fun card_gt_0_iff) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
296 |
end |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
297 |
|
48051 | 298 |
instantiation "fun" :: (card_UNIV, card_UNIV) card_UNIV begin |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
299 |
definition "card_UNIV = Phantom('a \<Rightarrow> 'b) |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
300 |
(let ca = of_phantom (card_UNIV :: 'a card_UNIV); |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
301 |
cb = of_phantom (card_UNIV :: 'b card_UNIV) |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
302 |
in if ca \<noteq> 0 \<and> cb \<noteq> 0 \<or> cb = 1 then cb ^ ca else 0)" |
48060 | 303 |
instance by intro_classes (simp add: card_UNIV_fun_def card_UNIV Let_def card_fun) |
304 |
end |
|
48051 | 305 |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
306 |
instantiation option :: (finite_UNIV) finite_UNIV begin |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
307 |
definition "finite_UNIV = Phantom('a option) (of_phantom (finite_UNIV :: 'a finite_UNIV))" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
308 |
instance by intro_classes (simp add: finite_UNIV_option_def finite_UNIV) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
309 |
end |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
310 |
|
48060 | 311 |
instantiation option :: (card_UNIV) card_UNIV begin |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
312 |
definition "card_UNIV = Phantom('a option) |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
313 |
(let c = of_phantom (card_UNIV :: 'a card_UNIV) in if c \<noteq> 0 then Suc c else 0)" |
48060 | 314 |
instance by intro_classes (simp add: card_UNIV_option_def card_UNIV card_UNIV_option) |
315 |
end |
|
48051 | 316 |
|
48060 | 317 |
instantiation String.literal :: card_UNIV begin |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
318 |
definition "finite_UNIV = Phantom(String.literal) False" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
319 |
definition "card_UNIV = Phantom(String.literal) 0" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
320 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
321 |
by intro_classes (simp_all add: card_UNIV_literal_def finite_UNIV_literal_def infinite_literal card_literal) |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
322 |
end |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
323 |
|
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
324 |
instantiation set :: (finite_UNIV) finite_UNIV begin |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
325 |
definition "finite_UNIV = Phantom('a set) (of_phantom (finite_UNIV :: 'a finite_UNIV))" |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
326 |
instance by intro_classes (simp add: finite_UNIV_set_def finite_UNIV Finite_Set.finite_set) |
48060 | 327 |
end |
328 |
||
329 |
instantiation set :: (card_UNIV) card_UNIV begin |
|
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
330 |
definition "card_UNIV = Phantom('a set) |
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
331 |
(let c = of_phantom (card_UNIV :: 'a card_UNIV) in if c = 0 then 0 else 2 ^ c)" |
48060 | 332 |
instance by intro_classes (simp add: card_UNIV_set_def card_UNIV_set card_UNIV) |
48051 | 333 |
end |
334 |
||
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52147
diff
changeset
|
335 |
lemma UNIV_finite_1: "UNIV = set [finite_1.a\<^sub>1]" |
48060 | 336 |
by(auto intro: finite_1.exhaust) |
337 |
||
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52147
diff
changeset
|
338 |
lemma UNIV_finite_2: "UNIV = set [finite_2.a\<^sub>1, finite_2.a\<^sub>2]" |
48060 | 339 |
by(auto intro: finite_2.exhaust) |
48051 | 340 |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52147
diff
changeset
|
341 |
lemma UNIV_finite_3: "UNIV = set [finite_3.a\<^sub>1, finite_3.a\<^sub>2, finite_3.a\<^sub>3]" |
48060 | 342 |
by(auto intro: finite_3.exhaust) |
48051 | 343 |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52147
diff
changeset
|
344 |
lemma UNIV_finite_4: "UNIV = set [finite_4.a\<^sub>1, finite_4.a\<^sub>2, finite_4.a\<^sub>3, finite_4.a\<^sub>4]" |
48060 | 345 |
by(auto intro: finite_4.exhaust) |
346 |
||
347 |
lemma UNIV_finite_5: |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52147
diff
changeset
|
348 |
"UNIV = set [finite_5.a\<^sub>1, finite_5.a\<^sub>2, finite_5.a\<^sub>3, finite_5.a\<^sub>4, finite_5.a\<^sub>5]" |
48060 | 349 |
by(auto intro: finite_5.exhaust) |
48051 | 350 |
|
48060 | 351 |
instantiation Enum.finite_1 :: card_UNIV begin |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
352 |
definition "finite_UNIV = Phantom(Enum.finite_1) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
353 |
definition "card_UNIV = Phantom(Enum.finite_1) 1" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
354 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
355 |
by intro_classes (simp_all add: UNIV_finite_1 card_UNIV_finite_1_def finite_UNIV_finite_1_def) |
48060 | 356 |
end |
357 |
||
358 |
instantiation Enum.finite_2 :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
359 |
definition "finite_UNIV = Phantom(Enum.finite_2) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
360 |
definition "card_UNIV = Phantom(Enum.finite_2) 2" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
361 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
362 |
by intro_classes (simp_all add: UNIV_finite_2 card_UNIV_finite_2_def finite_UNIV_finite_2_def) |
48060 | 363 |
end |
48051 | 364 |
|
48060 | 365 |
instantiation Enum.finite_3 :: card_UNIV begin |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
366 |
definition "finite_UNIV = Phantom(Enum.finite_3) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
367 |
definition "card_UNIV = Phantom(Enum.finite_3) 3" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
368 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
369 |
by intro_classes (simp_all add: UNIV_finite_3 card_UNIV_finite_3_def finite_UNIV_finite_3_def) |
48060 | 370 |
end |
371 |
||
372 |
instantiation Enum.finite_4 :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
373 |
definition "finite_UNIV = Phantom(Enum.finite_4) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
374 |
definition "card_UNIV = Phantom(Enum.finite_4) 4" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
375 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
376 |
by intro_classes (simp_all add: UNIV_finite_4 card_UNIV_finite_4_def finite_UNIV_finite_4_def) |
48060 | 377 |
end |
378 |
||
379 |
instantiation Enum.finite_5 :: card_UNIV begin |
|
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
380 |
definition "finite_UNIV = Phantom(Enum.finite_5) True" |
48164
e97369f20c30
change card_UNIV from itself to phantom type to avoid unnecessary closures in generated code
Andreas Lochbihler
parents:
48070
diff
changeset
|
381 |
definition "card_UNIV = Phantom(Enum.finite_5) 5" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
382 |
instance |
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
383 |
by intro_classes (simp_all add: UNIV_finite_5 card_UNIV_finite_5_def finite_UNIV_finite_5_def) |
48051 | 384 |
end |
385 |
||
60500 | 386 |
subsection \<open>Code setup for sets\<close> |
48051 | 387 |
|
60500 | 388 |
text \<open> |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
389 |
Implement @{term "CARD('a)"} via @{term card_UNIV} and provide |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
390 |
implementations for @{term "finite"}, @{term "card"}, @{term "op \<subseteq>"}, |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
391 |
and @{term "op ="}if the calling context already provides @{class finite_UNIV} |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
392 |
and @{class card_UNIV} instances. If we implemented the latter |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
393 |
always via @{term card_UNIV}, we would require instances of essentially all |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
394 |
element types, i.e., a lot of instantiation proofs and -- at run time -- |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
395 |
possibly slow dictionary constructions. |
60500 | 396 |
\<close> |
51116
0dac0158b8d4
implement code generation for finite, card, op = and op <= for sets always via finite_UNIV and card_UNIV, as fragile rewrites based on sorts are hard to find and debug
Andreas Lochbihler
parents:
49948
diff
changeset
|
397 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
398 |
context |
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
399 |
begin |
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
400 |
|
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
401 |
qualified definition card_UNIV' :: "'a card_UNIV" |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
402 |
where [code del]: "card_UNIV' = Phantom('a) CARD('a)" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
403 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
404 |
lemma CARD_code [code_unfold]: |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
405 |
"CARD('a) = of_phantom (card_UNIV' :: 'a card_UNIV)" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
406 |
by(simp add: card_UNIV'_def) |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
407 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
408 |
lemma card_UNIV'_code [code]: |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
409 |
"card_UNIV' = card_UNIV" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
410 |
by(simp add: card_UNIV card_UNIV'_def) |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
411 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
412 |
end |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
413 |
|
48051 | 414 |
lemma card_Compl: |
415 |
"finite A \<Longrightarrow> card (- A) = card (UNIV :: 'a set) - card (A :: 'a set)" |
|
416 |
by (metis Compl_eq_Diff_UNIV card_Diff_subset top_greatest) |
|
417 |
||
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
418 |
context fixes xs :: "'a :: finite_UNIV list" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
419 |
begin |
48062
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
420 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
421 |
qualified definition finite' :: "'a set \<Rightarrow> bool" |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
422 |
where [simp, code del, code_abbrev]: "finite' = finite" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
423 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
424 |
lemma finite'_code [code]: |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
425 |
"finite' (set xs) \<longleftrightarrow> True" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
426 |
"finite' (List.coset xs) \<longleftrightarrow> of_phantom (finite_UNIV :: 'a finite_UNIV)" |
48176
3d9c1ddb9f47
new type class for computing finiteness of types with instantiations
Andreas Lochbihler
parents:
48165
diff
changeset
|
427 |
by(simp_all add: card_gt_0_iff finite_UNIV) |
48062
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
428 |
|
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
429 |
end |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
430 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
431 |
context fixes xs :: "'a :: card_UNIV list" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
432 |
begin |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
433 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
434 |
qualified definition card' :: "'a set \<Rightarrow> nat" |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
435 |
where [simp, code del, code_abbrev]: "card' = card" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
436 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
437 |
lemma card'_code [code]: |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
438 |
"card' (set xs) = length (remdups xs)" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
439 |
"card' (List.coset xs) = of_phantom (card_UNIV :: 'a card_UNIV) - length (remdups xs)" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
440 |
by(simp_all add: List.card_set card_Compl card_UNIV) |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
441 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
442 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
443 |
qualified definition subset' :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
444 |
where [simp, code del, code_abbrev]: "subset' = op \<subseteq>" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
445 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
446 |
lemma subset'_code [code]: |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
447 |
"subset' A (List.coset ys) \<longleftrightarrow> (\<forall>y \<in> set ys. y \<notin> A)" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
448 |
"subset' (set ys) B \<longleftrightarrow> (\<forall>y \<in> set ys. y \<in> B)" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
449 |
"subset' (List.coset xs) (set ys) \<longleftrightarrow> (let n = CARD('a) in n > 0 \<and> card(set (xs @ ys)) = n)" |
48062
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
450 |
by(auto simp add: Let_def card_gt_0_iff dest: card_eq_UNIV_imp_eq_UNIV intro: arg_cong[where f=card]) |
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
451 |
(metis finite_compl finite_set rev_finite_subset) |
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
452 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
61076
diff
changeset
|
453 |
qualified definition eq_set :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
454 |
where [simp, code del, code_abbrev]: "eq_set = op =" |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
455 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
456 |
lemma eq_set_code [code]: |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
457 |
fixes ys |
48051 | 458 |
defines "rhs \<equiv> |
48059 | 459 |
let n = CARD('a) |
48051 | 460 |
in if n = 0 then False else |
461 |
let xs' = remdups xs; ys' = remdups ys |
|
462 |
in length xs' + length ys' = n \<and> (\<forall>x \<in> set xs'. x \<notin> set ys') \<and> (\<forall>y \<in> set ys'. y \<notin> set xs')" |
|
60583 | 463 |
shows "eq_set (List.coset xs) (set ys) \<longleftrightarrow> rhs" |
464 |
and "eq_set (set ys) (List.coset xs) \<longleftrightarrow> rhs" |
|
465 |
and "eq_set (set xs) (set ys) \<longleftrightarrow> (\<forall>x \<in> set xs. x \<in> set ys) \<and> (\<forall>y \<in> set ys. y \<in> set xs)" |
|
466 |
and "eq_set (List.coset xs) (List.coset ys) \<longleftrightarrow> (\<forall>x \<in> set xs. x \<in> set ys) \<and> (\<forall>y \<in> set ys. y \<in> set xs)" |
|
61166
5976fe402824
renamed method "goals" to "goal_cases" to emphasize its meaning;
wenzelm
parents:
61115
diff
changeset
|
467 |
proof goal_cases |
60583 | 468 |
{ |
469 |
case 1 |
|
470 |
show ?case (is "?lhs \<longleftrightarrow> ?rhs") |
|
471 |
proof |
|
472 |
show ?rhs if ?lhs |
|
473 |
using that |
|
474 |
by (auto simp add: rhs_def Let_def List.card_set[symmetric] |
|
475 |
card_Un_Int[where A="set xs" and B="- set xs"] card_UNIV |
|
476 |
Compl_partition card_gt_0_iff dest: sym)(metis finite_compl finite_set) |
|
477 |
show ?lhs if ?rhs |
|
478 |
proof - |
|
479 |
have "\<lbrakk> \<forall>y\<in>set xs. y \<notin> set ys; \<forall>x\<in>set ys. x \<notin> set xs \<rbrakk> \<Longrightarrow> set xs \<inter> set ys = {}" by blast |
|
480 |
with that show ?thesis |
|
481 |
by (auto simp add: rhs_def Let_def List.card_set[symmetric] |
|
482 |
card_UNIV card_gt_0_iff card_Un_Int[where A="set xs" and B="set ys"] |
|
62390 | 483 |
dest: card_eq_UNIV_imp_eq_UNIV split: if_split_asm) |
60583 | 484 |
qed |
485 |
qed |
|
486 |
} |
|
487 |
moreover |
|
488 |
case 2 |
|
489 |
ultimately show ?case unfolding eq_set_def by blast |
|
490 |
next |
|
491 |
case 3 |
|
492 |
show ?case unfolding eq_set_def List.coset_def by blast |
|
493 |
next |
|
494 |
case 4 |
|
495 |
show ?case unfolding eq_set_def List.coset_def by blast |
|
48051 | 496 |
qed |
497 |
||
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
498 |
end |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
499 |
|
60500 | 500 |
text \<open> |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
501 |
Provide more informative exceptions than Match for non-rewritten cases. |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
502 |
If generated code raises one these exceptions, then a code equation calls |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
503 |
the mentioned operator for an element type that is not an instance of |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
504 |
@{class card_UNIV} and is therefore not implemented via @{term card_UNIV}. |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
505 |
Constrain the element type with sort @{class card_UNIV} to change this. |
60500 | 506 |
\<close> |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
507 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
508 |
lemma card_coset_error [code]: |
53745 | 509 |
"card (List.coset xs) = |
510 |
Code.abort (STR ''card (List.coset _) requires type class instance card_UNIV'') |
|
511 |
(\<lambda>_. card (List.coset xs))" |
|
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
512 |
by(simp) |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
513 |
|
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
514 |
lemma coset_subseteq_set_code [code]: |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
515 |
"List.coset xs \<subseteq> set ys \<longleftrightarrow> |
53745 | 516 |
(if xs = [] \<and> ys = [] then False |
517 |
else Code.abort |
|
518 |
(STR ''subset_eq (List.coset _) (List.set _) requires type class instance card_UNIV'') |
|
519 |
(\<lambda>_. List.coset xs \<subseteq> set ys))" |
|
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
520 |
by simp |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
521 |
|
61585 | 522 |
notepad begin \<comment> "test code setup" |
51139
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
523 |
have "List.coset [True] = set [False] \<and> |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
524 |
List.coset [] \<subseteq> List.set [True, False] \<and> |
c8e3cf3520b3
partially revert 0dac0158b8d4 as it too aggressively spreads card_UNIV type class whose dictionary constructions can slow down generated code;
Andreas Lochbihler
parents:
51116
diff
changeset
|
525 |
finite (List.coset [True])" |
48062
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
526 |
by eval |
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
527 |
end |
9014e78ccde2
improved code setup for card, finite, subset
Andreas Lochbihler
parents:
48060
diff
changeset
|
528 |
|
48051 | 529 |
end |