aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-05-18 15:57:21 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-05-18 15:57:21 +0000
commitfaa0de5c67594980f8ad871dcf71c0dc98865a5e (patch)
treea95bd8204fbdeb0925ab64bd15992d4c35ce6f17 /kernel
parente7c9f5f130f5187e5d9b43c8f0ed15deb49e4b2c (diff)
Some ocamldoc comments + Fixing name of .coqrc.version file in refman
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13013 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/declarations.mli6
-rw-r--r--kernel/inductive.mli3
2 files changed, 4 insertions, 5 deletions
diff --git a/kernel/declarations.mli b/kernel/declarations.mli
index 3e8de34c4..36af9dc48 100644
--- a/kernel/declarations.mli
+++ b/kernel/declarations.mli
@@ -40,7 +40,7 @@ type constant_body = {
const_body : constr_substituted option;
const_type : constant_type;
const_body_code : to_patch_substituted;
- (*i const_type_code : to_patch;i*)
+ (* const_type_code : to_patch;*)
const_constraints : constraints;
const_opaque : bool;
const_inline : bool}
@@ -67,11 +67,11 @@ val recarg_length : wf_paths -> int -> int
val subst_wf_paths : substitution -> wf_paths -> wf_paths
(**
-{% \begin{verbatim} %}
+{v
Inductive I1 (params) : U1 := c11 : T11 | ... | c1p1 : T1p1
...
with In (params) : Un := cn1 : Tn1 | ... | cnpn : Tnpn
-{% \end{verbatim} %}
+v}
*)
type monomorphic_inductive_arity = {
diff --git a/kernel/inductive.mli b/kernel/inductive.mli
index 202b1aa4c..73bd2692e 100644
--- a/kernel/inductive.mli
+++ b/kernel/inductive.mli
@@ -89,8 +89,7 @@ val max_inductive_sort : sorts array -> universe
val instantiate_universes : env -> rel_context ->
polymorphic_arity -> types array -> rel_context * sorts
-(**************************************************************
- Debug *)
+(** {6 Debug} *)
type size = Large | Strict
type subterm_spec =