src/HOLCF/Fix.thy
changeset 16079 757e1c4a8081
parent 16070 4a83dd540b88
child 16082 ebb53ebfd4e2
--- a/src/HOLCF/Fix.thy	Wed May 25 16:14:40 2005 +0200
+++ b/src/HOLCF/Fix.thy	Thu May 26 00:30:24 2005 +0200
@@ -247,6 +247,18 @@
 apply assumption
 done
 
+text {* some lemmata for functions with flat/chfin domain/range types *}
+
+lemma adm_chfindom: "adm (%(u::'a::cpo->'b::chfin). P(u$s))"
+apply (unfold adm_def)
+apply (intro strip)
+apply (drule chfin_Rep_CFunR)
+apply (erule_tac x = "s" in allE)
+apply clarsimp
+done
+
+(* adm_flat not needed any more, since it is a special case of adm_chfindom *)
+
 text {* fixed point induction *}
 
 lemma fix_ind: