src/HOL/Library/Cset_Monad.thy
author huffman
Wed, 07 Dec 2011 10:50:30 +0100
changeset 45775 6c340de26a0d
parent 44898 ec3f30b8c78c
child 47232 e2f0176149d0
permissions -rw-r--r--
add cancellation simprocs for type enat

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