src/HOL/HOLCF/Sprod.thy
changeset 41430 1aa23e9f2c87
parent 40774 0437dbc127b3
child 41479 655f583840d0
--- a/src/HOL/HOLCF/Sprod.thy	Tue Jan 04 15:03:27 2011 -0800
+++ b/src/HOL/HOLCF/Sprod.thy	Tue Jan 04 15:32:56 2011 -0800
@@ -117,7 +117,7 @@
   "\<lbrakk>x \<noteq> \<bottom>; y \<noteq> \<bottom>; (:x, y:) = (:a, b:)\<rbrakk> \<Longrightarrow> x = a \<and> y = b"
 by (rule spair_eq [THEN iffD1])
 
-lemma inst_sprod_pcpo2: "UU = (:UU,UU:)"
+lemma inst_sprod_pcpo2: "\<bottom> = (:\<bottom>, \<bottom>:)"
 by simp
 
 lemma sprodE2: "(\<And>x y. p = (:x, y:) \<Longrightarrow> Q) \<Longrightarrow> Q"