src/HOLCF/IOA/meta_theory/Sequence.thy
changeset 3275 3f53f2c876f4
parent 3071 981258186b71
child 3952 dca1bce88ec8
equal deleted inserted replaced
3274:70939b0fadfb 3275:3f53f2c876f4
     1 (*  Title:      HOLCF/IOA/meta_theory/Sequence.thy
     1 (*  Title:      HOLCF/IOA/meta_theory/Sequence.thy
     2     ID:        
     2     ID:         $Id$
     3     Author:     Olaf M"uller
     3     Author:     Olaf M"uller
     4     Copyright   1996  TU Muenchen
     4     Copyright   1996  TU Muenchen
     5 
     5 
     6 Sequences over flat domains with lifted elements
     6 Sequences over flat domains with lifted elements
     7 
     7 
    81 
    81 
    82 (* for test purposes should be deleted FIX !! *)
    82 (* for test purposes should be deleted FIX !! *)
    83 adm_all    "adm f"
    83 adm_all    "adm f"
    84 
    84 
    85 
    85 
    86 take_reduction
       
    87   "[| Finite x; !! k. k < n ==> seq_take k`y1 = seq_take k`y2 |]
       
    88    ==> seq_take n`(x @@ (t>>y1)) =  seq_take n`(x @@ (t>>y2))"
       
    89 
       
    90 
       
    91 end
    86 end