# HG changeset patch # User haftmann # Date 1256285309 -7200 # Node ID 180feec9acf6a341dce24c2639cbef335dacff6d # Parent 06a48bbeb22a68bb18cf9ef54e4d072f5c825aa2 renamed f_inv_onto_f to f_inv_into_f (cf. 764547b68538) diff -r 06a48bbeb22a -r 180feec9acf6 src/HOLCF/Universal.thy --- a/src/HOLCF/Universal.thy Thu Oct 22 16:58:22 2009 +0200 +++ b/src/HOLCF/Universal.thy Fri Oct 23 10:08:29 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