| author | paulson <lp15@cam.ac.uk> | 
| Tue, 28 Apr 2015 16:23:05 +0100 | |
| changeset 60149 | 9b0825a00b1a | 
| parent 58881 | b9556a055632 | 
| child 60500 | 903bb1495239 | 
| permissions | -rw-r--r-- | 
| 35303 | 1 | (* Author: Florian Haftmann, TU Muenchen *) | 
| 2 | ||
| 58881 | 3 | section {* Lists with elements distinct as canonical example for datatype invariants *}
 | 
| 35303 | 4 | |
| 5 | theory Dlist | |
| 45990 
b7b905b23b2a
incorporated More_Set and More_List into the Main body -- to be consolidated later
 haftmann parents: 
45927diff
changeset | 6 | imports Main | 
| 35303 | 7 | begin | 
| 8 | ||
| 43146 | 9 | subsection {* The type of distinct lists *}
 | 
| 35303 | 10 | |
| 49834 | 11 | typedef 'a dlist = "{xs::'a list. distinct xs}"
 | 
| 35303 | 12 | morphisms list_of_dlist Abs_dlist | 
| 13 | proof | |
| 45694 
4a8743618257
prefer typedef without extra definition and alternative name;
 wenzelm parents: 
43764diff
changeset | 14 |   show "[] \<in> {xs. distinct xs}" by simp
 | 
| 35303 | 15 | qed | 
| 16 | ||
| 39380 
5a2662c1e44a
established emerging canonical names *_eqI and *_eq_iff
 haftmann parents: 
38857diff
changeset | 17 | lemma dlist_eq_iff: | 
| 
5a2662c1e44a
established emerging canonical names *_eqI and *_eq_iff
 haftmann parents: 
38857diff
changeset | 18 | "dxs = dys \<longleftrightarrow> list_of_dlist dxs = list_of_dlist dys" | 
| 
5a2662c1e44a
established emerging canonical names *_eqI and *_eq_iff
 haftmann parents: 
38857diff
changeset | 19 | by (simp add: list_of_dlist_inject) | 
| 36274 | 20 | |
| 39380 
5a2662c1e44a
established emerging canonical names *_eqI and *_eq_iff
 haftmann parents: 
38857diff
changeset | 21 | lemma dlist_eqI: | 
| 
5a2662c1e44a
established emerging canonical names *_eqI and *_eq_iff
 haftmann parents: 
38857diff
changeset | 22 | "list_of_dlist dxs = list_of_dlist dys \<Longrightarrow> dxs = dys" | 
| 
5a2662c1e44a
established emerging canonical names *_eqI and *_eq_iff
 haftmann parents: 
38857diff
changeset | 23 | by (simp add: dlist_eq_iff) | 
| 36112 
7fa17a225852
user interface for abstract datatypes is an attribute, not a command
 haftmann parents: 
35688diff
changeset | 24 | |
| 35303 | 25 | text {* Formal, totalized constructor for @{typ "'a dlist"}: *}
 | 
| 26 | ||
| 27 | definition Dlist :: "'a list \<Rightarrow> 'a dlist" where | |
| 37765 | 28 | "Dlist xs = Abs_dlist (remdups xs)" | 
| 35303 | 29 | |
| 39380 
5a2662c1e44a
established emerging canonical names *_eqI and *_eq_iff
 haftmann parents: 
38857diff
changeset | 30 | lemma distinct_list_of_dlist [simp, intro]: | 
| 35303 | 31 | "distinct (list_of_dlist dxs)" | 
| 32 | using list_of_dlist [of dxs] by simp | |
| 33 | ||
| 34 | lemma list_of_dlist_Dlist [simp]: | |
| 35 | "list_of_dlist (Dlist xs) = remdups xs" | |
| 36 | by (simp add: Dlist_def Abs_dlist_inverse) | |
| 37 | ||
| 39727 | 38 | lemma remdups_list_of_dlist [simp]: | 
| 39 | "remdups (list_of_dlist dxs) = list_of_dlist dxs" | |
| 40 | by simp | |
| 41 | ||
| 36112 
7fa17a225852
user interface for abstract datatypes is an attribute, not a command
 haftmann parents: 
35688diff
changeset | 42 | lemma Dlist_list_of_dlist [simp, code abstype]: | 
| 35303 | 43 | "Dlist (list_of_dlist dxs) = dxs" | 
| 44 | by (simp add: Dlist_def list_of_dlist_inverse distinct_remdups_id) | |
| 45 | ||
| 46 | ||
| 47 | text {* Fundamental operations: *}
 | |
| 48 | ||
| 49 | definition empty :: "'a dlist" where | |
| 50 | "empty = Dlist []" | |
| 51 | ||
| 52 | definition insert :: "'a \<Rightarrow> 'a dlist \<Rightarrow> 'a dlist" where | |
| 53 | "insert x dxs = Dlist (List.insert x (list_of_dlist dxs))" | |
| 54 | ||
| 55 | definition remove :: "'a \<Rightarrow> 'a dlist \<Rightarrow> 'a dlist" where | |
| 56 | "remove x dxs = Dlist (remove1 x (list_of_dlist dxs))" | |
| 57 | ||
| 58 | definition map :: "('a \<Rightarrow> 'b) \<Rightarrow> 'a dlist \<Rightarrow> 'b dlist" where
 | |
| 59 | "map f dxs = Dlist (remdups (List.map f (list_of_dlist dxs)))" | |
| 60 | ||
| 61 | definition filter :: "('a \<Rightarrow> bool) \<Rightarrow> 'a dlist \<Rightarrow> 'a dlist" where
 | |
| 62 | "filter P dxs = Dlist (List.filter P (list_of_dlist dxs))" | |
| 63 | ||
| 64 | ||
| 65 | text {* Derived operations: *}
 | |
| 66 | ||
| 67 | definition null :: "'a dlist \<Rightarrow> bool" where | |
| 68 | "null dxs = List.null (list_of_dlist dxs)" | |
| 69 | ||
| 70 | definition member :: "'a dlist \<Rightarrow> 'a \<Rightarrow> bool" where | |
| 71 | "member dxs = List.member (list_of_dlist dxs)" | |
| 72 | ||
| 73 | definition length :: "'a dlist \<Rightarrow> nat" where | |
| 74 | "length dxs = List.length (list_of_dlist dxs)" | |
| 75 | ||
| 76 | definition fold :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> 'a dlist \<Rightarrow> 'b \<Rightarrow> 'b" where
 | |
| 46133 
d9fe85d3d2cd
incorporated canonical fold combinator on lists into body of List theory; refactored passages on List.fold(l/r)
 haftmann parents: 
45990diff
changeset | 77 | "fold f dxs = List.fold f (list_of_dlist dxs)" | 
| 37022 
f9681d9d1d56
moved generic List operations to theory More_List
 haftmann parents: 
36980diff
changeset | 78 | |
| 
f9681d9d1d56
moved generic List operations to theory More_List
 haftmann parents: 
36980diff
changeset | 79 | definition foldr :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> 'a dlist \<Rightarrow> 'b \<Rightarrow> 'b" where
 | 
| 
f9681d9d1d56
moved generic List operations to theory More_List
 haftmann parents: 
36980diff
changeset | 80 | "foldr f dxs = List.foldr f (list_of_dlist dxs)" | 
| 35303 | 81 | |
| 82 | ||
| 43146 | 83 | subsection {* Executable version obeying invariant *}
 | 
| 35303 | 84 | |
| 85 | lemma list_of_dlist_empty [simp, code abstract]: | |
| 86 | "list_of_dlist empty = []" | |
| 87 | by (simp add: empty_def) | |
| 88 | ||
| 89 | lemma list_of_dlist_insert [simp, code abstract]: | |
| 90 | "list_of_dlist (insert x dxs) = List.insert x (list_of_dlist dxs)" | |
| 91 | by (simp add: insert_def) | |
| 92 | ||
| 93 | lemma list_of_dlist_remove [simp, code abstract]: | |
| 94 | "list_of_dlist (remove x dxs) = remove1 x (list_of_dlist dxs)" | |
| 95 | by (simp add: remove_def) | |
| 96 | ||
| 97 | lemma list_of_dlist_map [simp, code abstract]: | |
| 98 | "list_of_dlist (map f dxs) = remdups (List.map f (list_of_dlist dxs))" | |
| 99 | by (simp add: map_def) | |
| 100 | ||
| 101 | lemma list_of_dlist_filter [simp, code abstract]: | |
| 102 | "list_of_dlist (filter P dxs) = List.filter P (list_of_dlist dxs)" | |
| 103 | by (simp add: filter_def) | |
| 104 | ||
| 105 | ||
| 36980 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 106 | text {* Explicit executable conversion *}
 | 
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 107 | |
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 108 | definition dlist_of_list [simp]: | 
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 109 | "dlist_of_list = Dlist" | 
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 110 | |
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 111 | lemma [code abstract]: | 
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 112 | "list_of_dlist (dlist_of_list xs) = remdups xs" | 
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 113 | by simp | 
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 114 | |
| 
1a4cc941171a
added implementations of Fset.Set, Fset.Coset; do not delete code equations for relational operators on fsets
 haftmann parents: 
36274diff
changeset | 115 | |
| 38512 | 116 | text {* Equality *}
 | 
| 117 | ||
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
38512diff
changeset | 118 | instantiation dlist :: (equal) equal | 
| 38512 | 119 | begin | 
| 120 | ||
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
38512diff
changeset | 121 | definition "HOL.equal dxs dys \<longleftrightarrow> HOL.equal (list_of_dlist dxs) (list_of_dlist dys)" | 
| 38512 | 122 | |
| 123 | instance proof | |
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
38512diff
changeset | 124 | qed (simp add: equal_dlist_def equal list_of_dlist_inject) | 
| 38512 | 125 | |
| 126 | end | |
| 127 | ||
| 43764 | 128 | declare equal_dlist_def [code] | 
| 129 | ||
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
38512diff
changeset | 130 | lemma [code nbe]: | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
38512diff
changeset | 131 | "HOL.equal (dxs :: 'a::equal dlist) dxs \<longleftrightarrow> True" | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
38512diff
changeset | 132 | by (fact equal_refl) | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
38512diff
changeset | 133 | |
| 38512 | 134 | |
| 43146 | 135 | subsection {* Induction principle and case distinction *}
 | 
| 37106 | 136 | |
| 137 | lemma dlist_induct [case_names empty insert, induct type: dlist]: | |
| 138 | assumes empty: "P empty" | |
| 139 | assumes insrt: "\<And>x dxs. \<not> member dxs x \<Longrightarrow> P dxs \<Longrightarrow> P (insert x dxs)" | |
| 140 | shows "P dxs" | |
| 141 | proof (cases dxs) | |
| 142 | case (Abs_dlist xs) | |
| 143 | then have "distinct xs" and dxs: "dxs = Dlist xs" by (simp_all add: Dlist_def distinct_remdups_id) | |
| 144 | from `distinct xs` have "P (Dlist xs)" | |
| 39915 
ecf97cf3d248
turned distinct and sorted into inductive predicates: yields nice induction principles for free; more elegant proofs
 haftmann parents: 
39727diff
changeset | 145 | proof (induct xs) | 
| 37106 | 146 | case Nil from empty show ?case by (simp add: empty_def) | 
| 147 | next | |
| 40122 
1d8ad2ff3e01
dropped (almost) redundant distinct.induct rule; distinct_simps again named distinct.simps
 haftmann parents: 
39915diff
changeset | 148 | case (Cons x xs) | 
| 37106 | 149 | then have "\<not> member (Dlist xs) x" and "P (Dlist xs)" | 
| 37595 
9591362629e3
dropped ancient infix mem; refined code generation operations in List.thy
 haftmann parents: 
37473diff
changeset | 150 | by (simp_all add: member_def List.member_def) | 
| 37106 | 151 | with insrt have "P (insert x (Dlist xs))" . | 
| 40122 
1d8ad2ff3e01
dropped (almost) redundant distinct.induct rule; distinct_simps again named distinct.simps
 haftmann parents: 
39915diff
changeset | 152 | with Cons show ?case by (simp add: insert_def distinct_remdups_id) | 
| 37106 | 153 | qed | 
| 154 | with dxs show "P dxs" by simp | |
| 155 | qed | |
| 156 | ||
| 55913 | 157 | lemma dlist_case [cases type: dlist]: | 
| 158 | obtains (empty) "dxs = empty" | |
| 159 | | (insert) x dys where "\<not> member dys x" and "dxs = insert x dys" | |
| 37106 | 160 | proof (cases dxs) | 
| 161 | case (Abs_dlist xs) | |
| 162 | then have dxs: "dxs = Dlist xs" and distinct: "distinct xs" | |
| 163 | by (simp_all add: Dlist_def distinct_remdups_id) | |
| 55913 | 164 | show thesis | 
| 165 | proof (cases xs) | |
| 166 | case Nil with dxs | |
| 167 | have "dxs = empty" by (simp add: empty_def) | |
| 168 | with empty show ?thesis . | |
| 37106 | 169 | next | 
| 170 | case (Cons x xs) | |
| 171 | with dxs distinct have "\<not> member (Dlist xs) x" | |
| 172 | and "dxs = insert x (Dlist xs)" | |
| 37595 
9591362629e3
dropped ancient infix mem; refined code generation operations in List.thy
 haftmann parents: 
37473diff
changeset | 173 | by (simp_all add: member_def List.member_def insert_def distinct_remdups_id) | 
| 55913 | 174 | with insert show ?thesis . | 
| 37106 | 175 | qed | 
| 176 | qed | |
| 177 | ||
| 178 | ||
| 43146 | 179 | subsection {* Functorial structure *}
 | 
| 40603 | 180 | |
| 55467 
a5c9002bc54d
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
 blanchet parents: 
49834diff
changeset | 181 | functor map: map | 
| 41372 | 182 | by (simp_all add: List.map.id remdups_map_remdups fun_eq_iff dlist_eq_iff) | 
| 40603 | 183 | |
| 48282 | 184 | |
| 45927 
e0305e4f02c9
adding quickcheck generator for distinct lists; adding examples
 bulwahn parents: 
45694diff
changeset | 185 | subsection {* Quickcheck generators *}
 | 
| 
e0305e4f02c9
adding quickcheck generator for distinct lists; adding examples
 bulwahn parents: 
45694diff
changeset | 186 | |
| 46565 | 187 | quickcheck_generator dlist predicate: distinct constructors: empty, insert | 
| 40603 | 188 | |
| 48282 | 189 | |
| 37022 
f9681d9d1d56
moved generic List operations to theory More_List
 haftmann parents: 
36980diff
changeset | 190 | hide_const (open) member fold foldr empty insert remove map filter null member length fold | 
| 35303 | 191 | |
| 192 | end |