--- a/src/HOL/Main.thy Tue Sep 05 18:47:27 2000 +0200
+++ b/src/HOL/Main.thy Tue Sep 05 18:47:46 2000 +0200
@@ -4,7 +4,8 @@
theory Main = Map + String:
+(*actually belongs to theory List*)
lemmas [mono] = lists_mono
+lemmas [recdef_cong] = map_cong
end
-