src/HOLCF/Fixrec.thy
changeset 40327 1dfdbd66093a
parent 40322 707eb30e8a53
child 40502 8e92772bc0e8
--- a/src/HOLCF/Fixrec.thy	Fri Oct 29 16:51:40 2010 -0700
+++ b/src/HOLCF/Fixrec.thy	Fri Oct 29 17:15:28 2010 -0700
@@ -222,11 +222,11 @@
 by simp
 
 lemma def_cont_fix_eq:
-  "\<lbrakk>f \<equiv> fix\<cdot>(Abs_CFun F); cont F\<rbrakk> \<Longrightarrow> f = F f"
+  "\<lbrakk>f \<equiv> fix\<cdot>(Abs_cfun F); cont F\<rbrakk> \<Longrightarrow> f = F f"
 by (simp, subst fix_eq, simp)
 
 lemma def_cont_fix_ind:
-  "\<lbrakk>f \<equiv> fix\<cdot>(Abs_CFun F); cont F; adm P; P \<bottom>; \<And>x. P x \<Longrightarrow> P (F x)\<rbrakk> \<Longrightarrow> P f"
+  "\<lbrakk>f \<equiv> fix\<cdot>(Abs_cfun F); cont F; adm P; P \<bottom>; \<And>x. P x \<Longrightarrow> P (F x)\<rbrakk> \<Longrightarrow> P f"
 by (simp add: fix_ind)
 
 text {* lemma for proving rewrite rules *}