diff -r a9d6cf6de9a8 -r 99fe356cbbc2 src/HOLCF/Fix.thy --- a/src/HOLCF/Fix.thy Fri May 08 19:28:11 2009 +0100 +++ b/src/HOLCF/Fix.thy Fri May 08 16:19:51 2009 -0700 @@ -90,7 +90,7 @@ apply simp done -lemma fix_least_less: "F\x \ x \ fix\F \ x" +lemma fix_least_below: "F\x \ x \ fix\F \ x" apply (simp add: fix_def2) apply (rule is_lub_thelub) apply (rule chain_iterate) @@ -98,17 +98,17 @@ apply (induct_tac i) apply simp apply simp -apply (erule rev_trans_less) +apply (erule rev_below_trans) apply (erule monofun_cfun_arg) done lemma fix_least: "F\x = x \ fix\F \ x" -by (rule fix_least_less, simp) +by (rule fix_least_below, simp) lemma fix_eqI: assumes fixed: "F\x = x" and least: "\z. F\z = z \ x \ z" shows "fix\F = x" -apply (rule antisym_less) +apply (rule below_antisym) apply (rule fix_least [OF fixed]) apply (rule least [OF fix_eq [symmetric]]) done @@ -230,10 +230,10 @@ have "?y1 \ y" by (rule fix_least, simp add: F_y) hence "cfst\(F\\x, ?y1\) \ cfst\(F\\x, y\)" by (simp add: monofun_cfun) hence "cfst\(F\\x, ?y1\) \ x" using F_x by simp - hence 1: "?x \ x" by (simp add: fix_least_less) + hence 1: "?x \ x" by (simp add: fix_least_below) hence "csnd\(F\\?x, y\) \ csnd\(F\\x, y\)" by (simp add: monofun_cfun) hence "csnd\(F\\?x, y\) \ y" using F_y by simp - hence 2: "?y \ y" by (simp add: fix_least_less) + hence 2: "?y \ y" by (simp add: fix_least_below) show "\?x, ?y\ \ z" using z 1 2 by simp qed