aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-05-06 20:49:50 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-05-06 20:49:50 +0000
commit3a569247c5d9260e89ed5a4230468cb60f6f53a0 (patch)
tree5c1b29f1de1b3db05d41ac65d41976a5f9356f64
parent0d23af050fe3f93fb3aef907ec4febd6c8d0b32d (diff)
Fixing ocamldoc compilation.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16483 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--lib/iArray.mli2
-rw-r--r--lib/pp.mli2
-rw-r--r--pretyping/matching.mli2
-rw-r--r--proofs/pfedit.mli4
4 files changed, 5 insertions, 5 deletions
diff --git a/lib/iArray.mli b/lib/iArray.mli
index 9c28eb82b..a3789845e 100644
--- a/lib/iArray.mli
+++ b/lib/iArray.mli
@@ -71,7 +71,7 @@ val singleton : 'a -> 'a t
(** The singleton array. *)
val diff : 'a t -> (int * 'a) list -> 'a t
-(** [diff t [(i1, x1); ...; (in, xn)] create an array identical to [t] except on
+(** [diff t [(i1, x1); ...; (in, xn)]] create an array identical to [t] except on
indices [ik] that will contain [xk]. If the same index is present several
times on the diff, which value is chosen is undefined. *)
diff --git a/lib/pp.mli b/lib/pp.mli
index bc7441836..ccc6651ae 100644
--- a/lib/pp.mli
+++ b/lib/pp.mli
@@ -106,7 +106,7 @@ val std_logger : logger
val set_logger : logger -> unit
-(** {6 Feedback sent, even asynchronously, to the user interface *)
+(** {6 Feedback sent, even asynchronously, to the user interface} *)
(* This stuff should be available to most of the system, line msg_* above.
* But I'm unsure this is the right place, especially for the global edit_id.
diff --git a/pretyping/matching.mli b/pretyping/matching.mli
index 5ba68f26b..3501584c0 100644
--- a/pretyping/matching.mli
+++ b/pretyping/matching.mli
@@ -33,7 +33,7 @@ type bound_ident_map = (Id.t * Id.t) list
numbers given in the pattern *)
val matches : constr_pattern -> constr -> patvar_map
-(** [matches_head pat c] does the same as |matches pat c] but accepts
+(** [matches_head pat c] does the same as [matches pat c] but accepts
[pat] to match an applicative prefix of [c] *)
val matches_head : constr_pattern -> constr -> patvar_map
diff --git a/proofs/pfedit.mli b/proofs/pfedit.mli
index 090edde5a..4ca23e711 100644
--- a/proofs/pfedit.mli
+++ b/proofs/pfedit.mli
@@ -99,8 +99,8 @@ val cook_proof : (Proof.proof -> unit) ->
val set_xml_cook_proof : (goal_kind * Proof.proof -> unit) -> unit
(** {6 ... } *)
-(** [get_pftreestate ()] returns the current focused pending proof or
- @raise NoCurrentProof *)
+(** [get_pftreestate ()] returns the current focused pending proof.
+ @raise NoCurrentProof if there is no pending proof. *)
val get_pftreestate : unit -> Proof.proof