lemma is_empty_empty
authorhaftmann
Sun, 11 Apr 2010 16:51:06 +0200
changeset 36110 4ab91a42666a
parent 36109 1028cf8c0d1b
child 36111 5844017e31f8
lemma is_empty_empty
src/HOL/Library/Mapping.thy
--- a/src/HOL/Library/Mapping.thy	Sun Apr 11 16:51:05 2010 +0200
+++ b/src/HOL/Library/Mapping.thy	Sun Apr 11 16:51:06 2010 +0200
@@ -122,6 +122,10 @@
   "bulkload xs = tabulate [0..<length xs] (nth xs)"
   by (rule mapping_eqI) (simp add: expand_fun_eq)
 
+lemma is_empty_empty:
+  "is_empty m \<longleftrightarrow> m = Mapping Map.empty"
+  by (cases m) (simp add: is_empty_def)
+
 
 subsection {* Some technical code lemmas *}