diff -r f9b43d197d16 -r 080b755377c0 src/HOL/Wellfounded.thy --- a/src/HOL/Wellfounded.thy Tue May 04 08:55:39 2010 +0200 +++ b/src/HOL/Wellfounded.thy Tue May 04 08:55:43 2010 +0200 @@ -68,7 +68,7 @@ assumes lin: "OFCLASS('a::ord, linorder_class)" shows "OFCLASS('a::ord, wellorder_class)" using lin by (rule wellorder_class.intro) - (blast intro: wellorder_axioms.intro wf_induct_rule [OF wf]) + (blast intro: class.wellorder_axioms.intro wf_induct_rule [OF wf]) lemma (in wellorder) wf: "wf {(x, y). x < y}"