src/HOL/Main.thy
changeset 9876 a069795f1060
parent 9854 a1383b55ac05
child 10261 bb2f1e859177
--- a/src/HOL/Main.thy	Wed Sep 06 13:32:25 2000 +0200
+++ b/src/HOL/Main.thy	Wed Sep 06 16:54:12 2000 +0200
@@ -6,6 +6,6 @@
 
 (*actually belongs to theory List*)
 lemmas [mono] = lists_mono
-lemmas [recdef_cong] = map_cong 
+lemmas [recdef_cong] = map_cong
 
 end