# HG changeset patch # User huffman # Date 1287620722 25200 # Node ID e0f372e18f3e1c9d9a6ae3faebad8336caf9f5b0 # Parent 89381a2f8864469edad002e9c7fde2c376a80cb8 add lemma lub_eq_bottom_iff diff -r 89381a2f8864 -r e0f372e18f3e src/HOLCF/Pcpo.thy --- a/src/HOLCF/Pcpo.thy Wed Oct 20 16:19:25 2010 -0700 +++ b/src/HOLCF/Pcpo.thy Wed Oct 20 17:25:22 2010 -0700 @@ -223,18 +223,14 @@ lemma UU_I: "x \ \ \ x = \" by (subst eq_UU_iff) +lemma lub_eq_bottom_iff: "chain Y \ (\i. Y i) = \ \ (\i. Y i = \)" +by (simp only: eq_UU_iff lub_below_iff) + lemma chain_UU_I: "\chain Y; (\i. Y i) = \\ \ \i. Y i = \" -apply (rule allI) -apply (rule UU_I) -apply (erule subst) -apply (erule is_ub_thelub) -done +by (simp add: lub_eq_bottom_iff) lemma chain_UU_I_inverse: "\i::nat. Y i = \ \ (\i. Y i) = \" -apply (rule lub_chain_maxelem) -apply (erule spec) -apply simp -done +by simp lemma chain_UU_I_inverse2: "(\i. Y i) \ \ \ \i::nat. Y i \ \" by (blast intro: chain_UU_I_inverse)