src/HOL/HOLCF/FOCUS/Stream_adm.thy
changeset 43919 a7e4fb1a0502
parent 42151 4da4fc77664b
child 43921 e8511be08ddd
equal deleted inserted replaced
43903:1e2aa420c660 43919:a7e4fb1a0502
    72 apply ( rule exI)
    72 apply ( rule exI)
    73 apply ( rule slen_strict_mono)
    73 apply ( rule slen_strict_mono)
    74 apply (   erule spec)
    74 apply (   erule spec)
    75 apply (  assumption)
    75 apply (  assumption)
    76 apply ( assumption)
    76 apply ( assumption)
    77 apply (metis inat_ord_code(4) slen_infinite)
    77 apply (metis enat_ord_code(4) slen_infinite)
    78 done
    78 done
    79 
    79 
    80 (* should be without reference to stream length? *)
    80 (* should be without reference to stream length? *)
    81 lemma flatstream_admI: "[|(!!Y. [| Porder.chain Y; !i. P (Y i); 
    81 lemma flatstream_admI: "[|(!!Y. [| Porder.chain Y; !i. P (Y i); 
    82  !k. ? j. Fin k < #((Y j)::'a::flat stream)|] ==> P(LUB i. Y i))|]==> adm P"
    82  !k. ? j. Fin k < #((Y j)::'a::flat stream)|] ==> P(LUB i. Y i))|]==> adm P"