src/ZF/ex/Limit.thy
changeset 58318 f95754ca7082
parent 46822 95f1e700b712
child 59788 6f7b6adac439
equal deleted inserted replaced
58317:21fac057681e 58318:f95754ca7082
  1882                     nat_into_Ord)
  1882                     nat_into_Ord)
  1883 done
  1883 done
  1884 
  1884 
  1885 (* The following theorem is needed/useful due to type check for rel_cfI,
  1885 (* The following theorem is needed/useful due to type check for rel_cfI,
  1886    but also elsewhere.
  1886    but also elsewhere.
  1887    Look for occurences of rel_cfI, rel_DinfI, etc to evaluate the problem. *)
  1887    Look for occurrences of rel_cfI, rel_DinfI, etc to evaluate the problem. *)
  1888 
  1888 
  1889 lemma lam_Dinf_cont:
  1889 lemma lam_Dinf_cont:
  1890   "[| emb_chain(DD,ee); n \<in> nat |]
  1890   "[| emb_chain(DD,ee); n \<in> nat |]
  1891      ==> (\<lambda>x \<in> set(Dinf(DD,ee)). x`n) \<in> cont(Dinf(DD,ee),DD`n)"
  1891      ==> (\<lambda>x \<in> set(Dinf(DD,ee)). x`n) \<in> cont(Dinf(DD,ee),DD`n)"
  1892 apply (rule contI)
  1892 apply (rule contI)