src/HOL/UNITY/UNITY.thy
changeset 24147 edc90be09ac1
parent 16417 9bc16273c2d4
child 30198 922f944f03b2
--- a/src/HOL/UNITY/UNITY.thy	Fri Aug 03 16:28:25 2007 +0200
+++ b/src/HOL/UNITY/UNITY.thy	Fri Aug 03 20:19:41 2007 +0200
@@ -55,7 +55,7 @@
     "increasing f == \<Inter>z. stable {s. z \<le> f s}"
 
 
-text{*Perhaps equalities.ML shouldn't add this in the first place!*}
+text{*Perhaps HOL shouldn't add this in the first place!*}
 declare image_Collect [simp del]
 
 subsubsection{*The abstract type of programs*}
@@ -346,7 +346,7 @@
 lemma Int_Union_Union: "Union(B) \<inter> A = Union((%C. C \<inter> A)`B)"
 by blast
 
-text{*Needed for WF reasoning in WFair.ML*}
+text{*Needed for WF reasoning in WFair.thy*}
 
 lemma Image_less_than [simp]: "less_than `` {k} = greaterThan k"
 by blast