src/HOLCF/FOCUS/Fstream.thy
author wenzelm
Tue, 06 Sep 2005 21:51:17 +0200
changeset 17293 ecf182ccc3ca
parent 15188 9d57263faf9e
child 19759 2d0896653e7a
permissions -rw-r--r--
converted to Isar theory format;

(*  Title:      HOLCF/FOCUS/Fstream.thy
    ID:         $Id$
    Author:     David von Oheimb, TU Muenchen

FOCUS streams (with lifted elements)
###TODO: integrate Fstreams.thy
*)

header {* FOCUS flat streams *}

theory Fstream
imports Stream
begin

defaultsort type

types 'a fstream = "'a lift stream"

consts

  fscons        :: "'a     \<Rightarrow> 'a fstream \<rightarrow> 'a fstream"
  fsfilter      :: "'a set \<Rightarrow> 'a fstream \<rightarrow> 'a fstream"

syntax

  "@emptystream":: "'a fstream"                           ("<>")
  "@fscons"     :: "'a \<Rightarrow> 'a fstream \<Rightarrow> 'a fstream"       ("(_~>_)"    [66,65] 65)
  "@fsfilter"   :: "'a set \<Rightarrow> 'a fstream \<Rightarrow> 'a fstream"   ("(_'(C')_)" [64,63] 63)

syntax (xsymbols)

  "@fscons"     :: "'a \<Rightarrow> 'a fstream \<Rightarrow> 'a fstream"       ("(_\<leadsto>_)"
                                                                     [66,65] 65)
  "@fsfilter"   :: "'a set \<Rightarrow> 'a fstream \<Rightarrow> 'a fstream" ("(_\<copyright>_)"
                                                                     [64,63] 63)
translations

  "<>"    => "\<bottom>"
  "a~>s"  == "fscons a\<cdot>s"
  "A(C)s" == "fsfilter A\<cdot>s"

defs

  fscons_def:    "fscons a   \<equiv> \<Lambda> s. Def a && s"
  fsfilter_def:  "fsfilter A \<equiv> sfilter\<cdot>(flift2 (\<lambda>x. x\<in>A))"

ML {* use_legacy_bindings (the_context ()) *}

end