src/HOL/Library/Cset_Monad.thy
changeset 47232 e2f0176149d0
parent 44898 ec3f30b8c78c
--- a/src/HOL/Library/Cset_Monad.thy	Fri Mar 30 17:25:34 2012 +0200
+++ b/src/HOL/Library/Cset_Monad.thy	Fri Mar 30 18:56:02 2012 +0200
@@ -1,15 +0,0 @@
-(* 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
\ No newline at end of file