src/HOL/MiniML/Maybe.thy
author berghofe
Tue, 30 Sep 1997 12:49:16 +0200
changeset 3746 e832a36121ab
parent 2525 477c05586286
child 3842 b55686a7b22c
permissions -rw-r--r--
Modified some links.

(* Title:     HOL/MiniML/Maybe.thy
   ID:        $Id$
   Author:    Wolfgang Naraschewski and Tobias Nipkow
   Copyright  1996 TU Muenchen

Universal error monad.
*)

Maybe = Option + List +

constdefs
  option_bind :: ['a option, 'a => 'b option] => 'b option
  "option_bind m f == case m of None => None | Some r => f r"

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

end