src/HOL/Library/Cset_Monad.thy
author bulwahn
Thu, 01 Dec 2011 22:14:35 +0100
changeset 45724 1f5fc44254d7
parent 44898 ec3f30b8c78c
child 47232 e2f0176149d0
permissions -rw-r--r--
the simple exhaustive compilation also indicates if counterexample is potentially spurious;

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