src/HOLCF/Ssum.thy
changeset 40327 1dfdbd66093a
parent 40322 707eb30e8a53
child 40502 8e92772bc0e8
--- a/src/HOLCF/Ssum.thy	Fri Oct 29 16:51:40 2010 -0700
+++ b/src/HOLCF/Ssum.thy	Fri Oct 29 17:15:28 2010 -0700
@@ -120,11 +120,11 @@
 
 lemma compact_sinlD: "compact (sinl\<cdot>x) \<Longrightarrow> compact x"
 unfolding compact_def
-by (drule adm_subst [OF cont_Rep_CFun2 [where f=sinl]], simp)
+by (drule adm_subst [OF cont_Rep_cfun2 [where f=sinl]], simp)
 
 lemma compact_sinrD: "compact (sinr\<cdot>x) \<Longrightarrow> compact x"
 unfolding compact_def
-by (drule adm_subst [OF cont_Rep_CFun2 [where f=sinr]], simp)
+by (drule adm_subst [OF cont_Rep_cfun2 [where f=sinr]], simp)
 
 lemma compact_sinl_iff [simp]: "compact (sinl\<cdot>x) = compact x"
 by (safe elim!: compact_sinl compact_sinlD)