src/HOLCF/Porder.thy
changeset 17372 d73f67e90a95
parent 16318 45b12a01382f
child 17810 3bdf516d93d8
--- a/src/HOLCF/Porder.thy	Tue Sep 13 22:49:12 2005 +0200
+++ b/src/HOLCF/Porder.thy	Tue Sep 13 23:30:01 2005 +0200
@@ -265,6 +265,9 @@
 
 text {* the lub of a constant chain is the constant *}
 
+lemma chain_const: "chain (\<lambda>i. c)"
+by (simp add: chainI)
+
 lemma lub_const: "range(%x. c) <<| c"
 apply (blast dest: ub_rangeD intro: is_lubI ub_rangeI)
 done