src/HOL/Library/Dlist.thy
changeset 40603 963ee2331d20
parent 40122 1d8ad2ff3e01
child 40672 abd4e7358847
--- a/src/HOL/Library/Dlist.thy	Thu Nov 18 17:01:15 2010 +0100
+++ b/src/HOL/Library/Dlist.thy	Thu Nov 18 17:01:15 2010 +0100
@@ -173,6 +173,12 @@
 qed
 
 
+section {* Functorial structure *}
+
+type_mapper map
+  by (auto intro: dlist_eqI simp add: remdups_map_remdups comp_def)
+
+
 section {* Implementation of sets by distinct lists -- canonical! *}
 
 definition Set :: "'a dlist \<Rightarrow> 'a fset" where