src/HOL/Wellfounded_Relations.thy
changeset 11008 f7333f055ef6
parent 10213 01c2744a3786
child 11136 e34e7f6d9b57
--- a/src/HOL/Wellfounded_Relations.thy	Wed Jan 31 10:15:01 2001 +0100
+++ b/src/HOL/Wellfounded_Relations.thy	Wed Jan 31 10:15:55 2001 +0100
@@ -36,7 +36,7 @@
 "finite_psubset == {(A,B). A < B & finite B}"
 
 (* For rec_defs where the first n parameters stay unchanged in the recursive
-   call. See While for an application.
+   call. See Library/While_Combinator.thy for an application.
 *)
  same_fst :: "('a => bool) => ('a => ('b * 'b)set) => (('a*'b)*('a*'b))set"
 "same_fst P R == {((x',y'),(x,y)) . x'=x & P x & (y',y) : R x}"