diff options
| author | ppedrot | 2012-06-22 15:14:30 +0000 |
|---|---|---|
| committer | ppedrot | 2012-06-22 15:14:30 +0000 |
| commit | 6b45f2d36929162cf92272bb60c2c245d9a0ead3 (patch) | |
| tree | 93aa975697b7de73563c84773d99b4c65b92173b /lib/loc.mli | |
| parent | fea214f82954197d23fda9a0e4e7d93e0cbf9b4c (diff) | |
Added an indirection with respect to Loc in Compat. As many [open Compat]
were closed (i.e. the only remaining ones are those of printing/parsing).
Meanwhile, a simplified interface is provided in loc.mli.
This also permits to put Pp in Clib, because it does not depend on
CAMLP4/5 anymore.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15475 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'lib/loc.mli')
| -rw-r--r-- | lib/loc.mli | 44 |
1 files changed, 44 insertions, 0 deletions
diff --git a/lib/loc.mli b/lib/loc.mli new file mode 100644 index 0000000000..c8e0901e9d --- /dev/null +++ b/lib/loc.mli @@ -0,0 +1,44 @@ +(************************************************************************) +(* v * The Coq Proof Assistant / The Coq Development Team *) +(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2010 *) +(* \VV/ **************************************************************) +(* // * This file is distributed under the terms of the *) +(* * GNU Lesser General Public License Version 2.1 *) +(************************************************************************) + +(** {5 Basic types} *) + +type t = Compat.Loc.t + +exception Exc_located of t * exn + +type 'a located = t * 'a + +(** {5 Location manipulation} *) + +(** This is inherited from CAMPL4/5. *) + +val unloc : t -> int * int +val make_loc : int * int -> t +val ghost : t +val merge : t -> t -> t +val raise : t -> exn -> 'a + +(** {5 Location utilities} *) + +val located_fold_left : ('a -> 'b -> 'a) -> 'a -> 'b located -> 'a +val located_iter2 : ('a -> 'b -> unit) -> 'a located -> 'b located -> unit + +val down_located : ('a -> 'b) -> 'a located -> 'b +(** Projects out a located object *) + +val pr_located : ('a -> Pp.std_ppcmds) -> 'a located -> Pp.std_ppcmds +(** Prints an object surrounded by its commented location *) + +(** {5 Backward compatibility} *) + +val dummy_loc : t +(** Same as [ghost] *) + +val join_loc : t -> t -> t +(** Same as [merge] *) |
