diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2005-01-21 17:18:23 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2005-01-21 17:18:23 +0000 |
commit | d7b2414b631d71e89e677d650b84bd4fadd44895 (patch) | |
tree | 47b653e7e0ae9b83dbc8a96b2c5be4717b2eefbd /kernel | |
parent | ea6bd4e5496f0fd7e059cd9b924f29ca80a38ae2 (diff) |
Compatibilité ocamlweb pour cible doc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@6616 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r-- | kernel/declarations.mli | 10 | ||||
-rw-r--r-- | kernel/environ.mli | 2 | ||||
-rw-r--r-- | kernel/inductive.mli | 2 | ||||
-rw-r--r-- | kernel/modops.mli | 2 |
4 files changed, 8 insertions, 8 deletions
diff --git a/kernel/declarations.mli b/kernel/declarations.mli index 30c0ffde0..3c99b67ac 100644 --- a/kernel/declarations.mli +++ b/kernel/declarations.mli @@ -33,7 +33,7 @@ type constant_body = { const_body : constr_substituted option; const_type : types; const_body_code : to_patch_substituted; - (* const_type_code : to_patch;*) + (*i const_type_code : to_patch;i*) const_constraints : constraints; const_opaque : bool } @@ -119,8 +119,8 @@ and module_specification_body = { msb_modtype : module_type_body; msb_equiv : module_path option; msb_constraints : constraints } - (* type_of(equiv) <: modtype (if given) - + substyping of past With_Module mergers *) + (* [type_of](equiv) <: modtype (if given) + + substyping of past [With_Module] mergers *) type structure_elem_body = @@ -136,7 +136,7 @@ and module_expr_body = | MEBfunctor of mod_bound_id * module_type_body * module_expr_body | MEBstruct of mod_self_id * module_structure_body | MEBapply of module_expr_body * module_expr_body (* (F A) *) - * constraints (* type_of(A) <: input_type_of(F) *) + * constraints (* [type_of](A) <: [input_type_of](F) *) and module_body = { mod_expr : module_expr_body option; @@ -144,7 +144,7 @@ and module_body = mod_type : module_type_body; mod_equiv : module_path option; mod_constraints : constraints } - (* type_of(mod_expr) <: mod_user_type (if given) *) + (* [type_of(mod_expr)] <: [mod_user_type] (if given) *) (* if equiv given then constraints are empty *) diff --git a/kernel/environ.mli b/kernel/environ.mli index 5be23b490..20027d32a 100644 --- a/kernel/environ.mli +++ b/kernel/environ.mli @@ -46,7 +46,7 @@ val engagement : env -> engagement option val empty_context : env -> bool (************************************************************************) -(*s Context of de Bruijn variables (rel_context) *) +(*s Context of de Bruijn variables ([rel_context]) *) val push_rel : rel_declaration -> env -> env val push_rel_context : rel_context -> env -> env val push_rec_types : rec_declaration -> env -> env diff --git a/kernel/inductive.mli b/kernel/inductive.mli index 0174b8020..f419bc3fa 100644 --- a/kernel/inductive.mli +++ b/kernel/inductive.mli @@ -62,7 +62,7 @@ val type_case_branches : given inductive type. *) val check_case_info : env -> inductive -> case_info -> unit -(* Find the ultimate inductive in the mind_equiv chain *) +(* Find the ultimate inductive in the [mind_equiv] chain *) val scrape_mind : env -> mutual_inductive -> mutual_inductive diff --git a/kernel/modops.mli b/kernel/modops.mli index 052bac243..f102a5b2c 100644 --- a/kernel/modops.mli +++ b/kernel/modops.mli @@ -42,7 +42,7 @@ val subst_signature_msid : module_signature_body -> module_signature_body (* [add_signature mp sign env] assumes that the substitution [msid] - \mapsto [mp] has already been performed (or is not necessary, like + $\mapsto$ [mp] has already been performed (or is not necessary, like when [mp = MPself msid]) *) val add_signature : module_path -> module_signature_body -> env -> env |