aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proofview_monad.mli
diff options
context:
space:
mode:
authorGravatar Arnaud Spiwack <arnaud@spiwack.net>2014-10-21 15:58:16 +0200
committerGravatar Arnaud Spiwack <arnaud@spiwack.net>2014-10-22 07:31:45 +0200
commitaab7ae42b7ed4a071a79600a1adf5a81bafb5f89 (patch)
treecbb2fc770f0105f64a12f1e0f461e02ff7408ae0 /proofs/proofview_monad.mli
parente33d2962b549e3b0930b00933bbd2dc29fd3a905 (diff)
Make names in [Proofview_monad] more uniform.
ret -> return, bind -> (>>=), etc… So that monads expose a [Monad.S] signature. Also Proofview now exposes the [Monad.S] signature directly rather than in a [Monad.S] subdirectory.
Diffstat (limited to 'proofs/proofview_monad.mli')
-rw-r--r--proofs/proofview_monad.mli19
1 files changed, 6 insertions, 13 deletions
diff --git a/proofs/proofview_monad.mli b/proofs/proofview_monad.mli
index 675b4c768..c1315e9f5 100644
--- a/proofs/proofview_monad.mli
+++ b/proofs/proofview_monad.mli
@@ -41,20 +41,17 @@ exception TacticFailure of exn
operations and require little documentation. *)
module NonLogical : sig
- type +'a t
- type 'a ref
+ include Monad.S
- val ret : 'a -> 'a t
- val bind : 'a t -> ('a -> 'b t) -> 'b t
- val map : ('a -> 'b) -> 'a t -> 'b t
val ignore : 'a t -> unit t
- val seq : unit t -> 'a t -> 'a t
+
+ type 'a ref
val ref : 'a -> 'a ref t
(** [Pervasives.(:=)] *)
- val set : 'a ref -> 'a -> unit t
+ val (:=) : 'a ref -> 'a -> unit t
(** [Pervasives.(!)] *)
- val get : 'a ref -> 'a t
+ val (!) : 'a ref -> 'a t
val read_line : string t
val print_char : char -> unit t
@@ -125,13 +122,9 @@ end
module Logical (P:Param) : sig
- type +'a t
+ include Monad.S
- val ret : 'a -> 'a t
- val bind : 'a t -> ('a -> 'b t) -> 'b t
- val map : ('a -> 'b) -> 'a t -> 'b t
val ignore : 'a t -> unit t
- val seq : unit t -> 'a t -> 'a t
val set : P.s -> unit t
val get : P.s t