src/HOL/W0/Maybe.thy
author nipkow
Fri, 17 Jan 1997 13:21:54 +0100
changeset 2518 bee082efaa46
child 2520 aecaa76e7eff
permissions -rw-r--r--
This is the old version og MiniML for the monomorphic case. The new version is now in MiniML.

(* Title:     HOL/MiniML/Maybe.thy
   ID:        $Id$
   Author:    Dieter Nazareth and Tobias Nipkow
   Copyright  1995 TU Muenchen

Universal error monad.
*)

Maybe = List +

datatype 'a maybe =  Ok 'a | Fail

constdefs
  bind :: ['a maybe, 'a => 'b maybe] => 'b maybe (infixl 60)
  "m bind f == case m of Ok r => f r | Fail => Fail"

syntax "@bind" :: [pttrns,'a maybe,'b] => 'c ("(_ := _;//_)" 0)
translations "P := E; F" == "E bind (%P.F)"

end