src/HOL/Library/Mapping.thy
changeset 40968 a6fcd305f7dc
parent 40605 0bc28f978bcf
child 41372 551eb49a6e91
equal deleted inserted replaced
40965:54b6c9e1c157 40968:a6fcd305f7dc
    48 
    48 
    49 lemma lookup_map [simp]:
    49 lemma lookup_map [simp]:
    50   "lookup (map f g m) = Option.map g \<circ> lookup m \<circ> f"
    50   "lookup (map f g m) = Option.map g \<circ> lookup m \<circ> f"
    51   by (simp add: map_def)
    51   by (simp add: map_def)
    52 
    52 
    53 type_mapper map
    53 type_lifting map
    54   by (auto intro!: mapping_eqI ext simp add: Option.map.compositionality Option.map.identity)
    54   by (auto intro!: mapping_eqI ext simp add: Option.map.compositionality Option.map.identity)
    55 
    55 
    56 
    56 
    57 subsection {* Derived operations *}
    57 subsection {* Derived operations *}
    58 
    58