src/HOL/Library/Cset_Monad.thy
author wenzelm
Thu, 16 Feb 2012 22:53:24 +0100
changeset 46507 1b24c24017dd
parent 44898 ec3f30b8c78c
child 47232 e2f0176149d0
permissions -rw-r--r--
tuned proofs;

(* Title: HOL/Library/Cset_Monad.thy
   Author: Andreas Lochbihler, Karlsruhe Institute of Technology
*)

header {* Monad notation for computable sets (cset) *}

theory Cset_Monad
imports Cset Monad_Syntax 
begin

setup {*
  Adhoc_Overloading.add_variant @{const_name bind} @{const_name Cset.bind}
*}

end