src/HOL/Map.ML
changeset 13890 90611b4e0054
parent 13811 f39f67982854
--- a/src/HOL/Map.ML	Tue Apr 01 16:08:34 2003 +0200
+++ b/src/HOL/Map.ML	Tue Apr 01 17:43:10 2003 +0200
@@ -8,17 +8,13 @@
 
 section "empty";
 
-Goalw [empty_def] "empty k = None";
-by (Simp_tac 1);
-qed "empty_def2";
-Addsimps [empty_def2];
-
 Goal "empty(x := None) = empty";
 by (rtac ext 1);
 by (Simp_tac 1);
 qed "empty_upd_none";
 Addsimps [empty_upd_none];
 
+(* FIXME: what is this sum_case nonsense?? *)
 Goal "sum_case empty empty = empty";
 by (rtac ext 1);
 by (simp_tac (simpset() addsplits [sum.split]) 1);
@@ -48,6 +44,7 @@
 qed "finite_range_updI";
 
 
+(* FIXME: what is this sum_case nonsense?? *)
 section "sum_case and empty/map_upd";
 
 Goal "sum_case (m(k|->y)) empty =  (sum_case m empty)(Inl k|->y)";