src/HOLCF/explicit_domains/Stream2.thy
author paulson
Tue, 16 Jul 1996 15:49:46 +0200
changeset 1868 836950047d85
parent 1479 21eb5e156d91
child 2569 3a8604f408c9
permissions -rw-r--r--
Put in minimal simpset to avoid excessive simplification, just as in revision 1.9 of HOL/indrule.ML

(* 
    ID:         $Id$
    Author:     Franz Regensburger
    Copyright   1993 Technische Universitaet Muenchen

Additional constants for stream
*)

Stream2 = Stream +

consts

smap            :: "('a -> 'b) -> 'a stream -> 'b stream"

defs

smap_def
  "smap == fix`(LAM h f s. stream_when`(LAM x l.scons `(f`x) `(h`f`l)) `s)"


end
      

(*
                smap`f`UU = UU
      x~=UU --> smap`f`(scons`x`xs) = scons `(f`x) `(smap`f`xs)

*)