src/HOL/Library/Cset_Monad.thy
author bulwahn
Tue, 10 Jan 2012 15:48:10 +0100
changeset 46171 19f68d7671f0
parent 44898 ec3f30b8c78c
child 47232 e2f0176149d0
permissions -rw-r--r--
proper hiding of facts and constants in AList_Impl and AList theory

(* 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