# HG changeset patch # User wenzelm # Date 1256219412 -7200 # Node ID 362f59fe50928b436ea250f785dfaee97fb0790d # Parent c39f6bd5a46b1799816646db058ec166a574f273 renamed f_inv_onto_f to f_inv_into_f (cf. 764547b68538); diff -r c39f6bd5a46b -r 362f59fe5092 src/HOLCF/Universal.thy --- a/src/HOLCF/Universal.thy Thu Oct 22 15:26:15 2009 +0200 +++ b/src/HOLCF/Universal.thy Thu Oct 22 15:50:12 2009 +0200 @@ -805,7 +805,7 @@ lemma basis_emb_prj_less: "ubasis_le (basis_emb (basis_prj x)) x" unfolding basis_prj_def - apply (subst f_inv_onto_f [where f=basis_emb]) + apply (subst f_inv_into_f [where f=basis_emb]) apply (rule ubasis_until) apply (rule range_eqI [where x=compact_bot]) apply simp