author | haftmann |
Fri, 14 Nov 2008 08:50:08 +0100 | |
changeset 28790 | 2efba7b18c5b |
parent 28789 | 5a404273ea8f |
child 28791 | cc16be808796 |
src/HOL/Map.thy | file | annotate | diff | comparison | revisions |
--- a/src/HOL/Map.thy Fri Nov 14 08:50:07 2008 +0100 +++ b/src/HOL/Map.thy Fri Nov 14 08:50:08 2008 +0100 @@ -509,6 +509,15 @@ \<exists>x. f x = None" by(bestsimp dest:ex_new_if_finite) +lemma dom_minus: + "f x = None \<Longrightarrow> dom f - insert x A = dom f - A" + unfolding dom_def by simp + +lemma insert_dom: + "f x = Some y \<Longrightarrow> insert x (dom f) = dom f" + unfolding dom_def by auto + + subsection {* @{term [source] ran} *} lemma ranI: "m a = Some b ==> b : ran m"