src/HOL/Library/Mapping.thy
changeset 55467 a5c9002bc54d
parent 55466 786edc984c98
child 55525 70b7e91fa1f9
equal deleted inserted replaced
55466:786edc984c98 55467:a5c9002bc54d
   108   "\<lambda>f g m. (map_option g \<circ> m \<circ> f)" parametric map_transfer .
   108   "\<lambda>f g m. (map_option g \<circ> m \<circ> f)" parametric map_transfer .
   109 
   109 
   110 
   110 
   111 subsection {* Functorial structure *}
   111 subsection {* Functorial structure *}
   112 
   112 
   113 enriched_type map: map
   113 functor map: map
   114   by (transfer, auto simp add: fun_eq_iff option.map_comp option.map_id)+
   114   by (transfer, auto simp add: fun_eq_iff option.map_comp option.map_id)+
   115 
   115 
   116 
   116 
   117 subsection {* Derived operations *}
   117 subsection {* Derived operations *}
   118 
   118