aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proofview_monad.mli
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-11-02 15:38:50 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-11-02 15:38:50 +0000
commit4da1a1e094a08a35d9de5fd0be373edc01ea18d5 (patch)
tree80fd123a61ec0add5b25f7ee36c32567105366b1 /proofs/proofview_monad.mli
parentaf63420fe7202f01b483812bc1f5ff50c5a640e2 (diff)
A dedicated view type for Proofview_gen.split.
It doesn't seem to affect performances. But the generated code is slightly cleaner. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@17005 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/proofview_monad.mli')
-rw-r--r--proofs/proofview_monad.mli5
1 files changed, 4 insertions, 1 deletions
diff --git a/proofs/proofview_monad.mli b/proofs/proofview_monad.mli
index bdebe658c..f9854ae0c 100644
--- a/proofs/proofview_monad.mli
+++ b/proofs/proofview_monad.mli
@@ -1,6 +1,9 @@
(* This is an interface for the code extracted from bootstrap/Monad.v.
The relevant comments are overthere. *)
+type ('a, 'b) list_view =
+| Nil of exn
+| Cons of 'a * 'b
type proofview = { initial : (Term.constr * Term.types) list;
solution : Evd.evar_map; comb : Goal.goal list }
@@ -58,7 +61,7 @@ module Logical : sig
val zero : exn -> 'a t
val plus : 'a t -> (exn -> 'a t) -> 'a t
- val split : 'a t -> (('a*(exn->'a t),exn) Util.union) t
+ val split : 'a t -> (('a,(exn->'a t)) list_view) t
val lift : 'a NonLogical.t -> 'a t