src/HOL/Library/Dlist.thy
changeset 40968 a6fcd305f7dc
parent 40672 abd4e7358847
child 41372 551eb49a6e91
equal deleted inserted replaced
40965:54b6c9e1c157 40968:a6fcd305f7dc
   173 qed
   173 qed
   174 
   174 
   175 
   175 
   176 section {* Functorial structure *}
   176 section {* Functorial structure *}
   177 
   177 
   178 type_mapper map
   178 type_lifting map
   179   by (auto intro: dlist_eqI simp add: remdups_map_remdups comp_def)
   179   by (auto intro: dlist_eqI simp add: remdups_map_remdups comp_def)
   180 
   180 
   181 
   181 
   182 section {* Implementation of sets by distinct lists -- canonical! *}
   182 section {* Implementation of sets by distinct lists -- canonical! *}
   183 
   183