src/HOL/Library/Cset_Monad.thy
changeset 48103 e2f0176149d0
parent 45769 ec3f30b8c78c
     1.1 --- a/src/HOL/Library/Cset_Monad.thy	Fri Mar 30 17:25:34 2012 +0200
     1.2 +++ b/src/HOL/Library/Cset_Monad.thy	Fri Mar 30 18:56:02 2012 +0200
     1.3 @@ -1,15 +0,0 @@
     1.4 -(* Title: HOL/Library/Cset_Monad.thy
     1.5 -   Author: Andreas Lochbihler, Karlsruhe Institute of Technology
     1.6 -*)
     1.7 -
     1.8 -header {* Monad notation for computable sets (cset) *}
     1.9 -
    1.10 -theory Cset_Monad
    1.11 -imports Cset Monad_Syntax 
    1.12 -begin
    1.13 -
    1.14 -setup {*
    1.15 -  Adhoc_Overloading.add_variant @{const_name bind} @{const_name Cset.bind}
    1.16 -*}
    1.17 -
    1.18 -end
    1.19 \ No newline at end of file