src/ZF/UNITY/Distributor.thy
changeset 14077 37c964462747
parent 14072 f932be305381
child 14095 a1ba833d6b61
--- a/src/ZF/UNITY/Distributor.thy	Fri Jun 27 13:15:40 2003 +0200
+++ b/src/ZF/UNITY/Distributor.thy	Fri Jun 27 18:40:25 2003 +0200
@@ -158,8 +158,9 @@
 apply (auto simp add: distr_spec_def distr_follows_def)
 apply (drule guaranteesD, assumption)
 apply (simp_all cong add: Follows_cong
-    add: refl_prefix
-       mono_bag_of [THEN subset_Follows_comp, THEN subsetD, unfolded comp_def])
+		add: refl_prefix
+		   mono_bag_of [THEN subset_Follows_comp, THEN subsetD, 
+				unfolded metacomp_def])
 done
 
 end