src/HOL/Library/Cset_Monad.thy
changeset 43976 af17d7934116
child 44898 ec3f30b8c78c
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Library/Cset_Monad.thy	Tue Jul 26 10:49:34 2011 +0200
@@ -0,0 +1,13 @@
+(* Author: Andreas Lochbihler, KIT *)
+
+header {* Add monad syntax for Csets *}
+
+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