changeset 17585 | f12d7ac88eb4 |
parent 16917 | 1fe50b19daba |
child 17816 | 9942c5ed866a |
--- a/src/HOLCF/Fix.thy Thu Sep 22 18:59:41 2005 +0200 +++ b/src/HOLCF/Fix.thy Thu Sep 22 19:06:05 2005 +0200 @@ -228,7 +228,7 @@ text {* computational induction for weak admissible formulae *} -lemma wfix_ind: "\<lbrakk>admw P; \<forall>n. P (iterate n F UU)\<rbrakk> \<Longrightarrow> P (fix\<cdot>F)" +lemma wfix_ind: "\<lbrakk>admw P; \<forall>n. P (iterate n F \<bottom>)\<rbrakk> \<Longrightarrow> P (fix\<cdot>F)" by (simp add: fix_def2 admw_def) lemma def_wfix_ind: