src/HOL/HOLCF/Bifinite.thy
changeset 41430 1aa23e9f2c87
parent 41413 64cd30d6b0b8
child 42151 4da4fc77664b
--- a/src/HOL/HOLCF/Bifinite.thy	Tue Jan 04 15:03:27 2011 -0800
+++ b/src/HOL/HOLCF/Bifinite.thy	Tue Jan 04 15:32:56 2011 -0800
@@ -253,7 +253,7 @@
 qed
 
 lemma approx_chain_unit: "approx_chain (\<bottom> :: nat \<Rightarrow> unit \<rightarrow> unit)"
-by (simp add: approx_chain_def cfun_eq_iff finite_deflation_UU)
+by (simp add: approx_chain_def cfun_eq_iff finite_deflation_bottom)
 
 instance unit :: bifinite
   by default (fast intro!: approx_chain_unit)