diff options
| author | filliatr | 2000-07-25 17:29:20 +0000 |
|---|---|---|
| committer | filliatr | 2000-07-25 17:29:20 +0000 |
| commit | c330f60f1617afcb42cebe2fd2ccf9f330ea4f89 (patch) | |
| tree | 53e61f40e19ea35216091af7324a6bbd4fc7e4bd /proofs | |
| parent | 968d65c616127446c5f1c5d3485e9efdc420e6a4 (diff) | |
retablissement make doc et make minicoq
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@571 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
| -rw-r--r-- | proofs/logic.mli | 17 | ||||
| -rw-r--r-- | proofs/tacinterp.mli | 2 | ||||
| -rw-r--r-- | proofs/tacmach.mli | 2 |
3 files changed, 10 insertions, 11 deletions
diff --git a/proofs/logic.mli b/proofs/logic.mli index dd27797254..9247d4ff6e 100644 --- a/proofs/logic.mli +++ b/proofs/logic.mli @@ -10,20 +10,19 @@ open Environ open Proof_type (*i*) -(* This suppresses check done in prim_refiner for the tactic given in +(* This suppresses check done in [prim_refiner] for the tactic given in argument; works by side-effect *) val without_check : tactic -> tactic -(* without_check respectively means:\\ -\\ - Intro: no check that the name does not exist\\ - Intro_after: no check that the name does not exist and that variables in +(* [without_check] respectively means:\\ + [Intro]: no check that the name does not exist\\ + [Intro_after]: no check that the name does not exist and that variables in its type does not escape their scope\\ - Intro_replacing: no check that the name does not exist and that variables in - its type does not escape their scope\\ - - Convert_hyp: no check that the name exist and that its type is convertible\\ + [Intro_replacing]: no check that the name does not exist and that + variables in its type does not escape their scope\\ + [Convert_hyp]: + no check that the name exist and that its type is convertible\\ *) (* The primitive refiner. *) diff --git a/proofs/tacinterp.mli b/proofs/tacinterp.mli index 39351dc1e5..50b454df8f 100644 --- a/proofs/tacinterp.mli +++ b/proofs/tacinterp.mli @@ -37,7 +37,7 @@ val val_interp : interp_sign -> Coqast.t -> value val interp_tacarg : interp_sign -> Coqast.t -> tactic_arg val interp : Coqast.t -> tactic -(*val vernac_interp : Coqast.t -> tactic*) +(*i val vernac_interp : Coqast.t -> tactic i*) val vernac_interp_atomic : identifier -> tactic_arg list -> tactic val is_just_undef_macro : Coqast.t -> string option diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli index 6ae4f9ae26..bf2b0a3bab 100644 --- a/proofs/tacmach.mli +++ b/proofs/tacmach.mli @@ -34,7 +34,7 @@ val apply_sig_tac : val pf_concl : goal sigma -> constr val pf_env : goal sigma -> env val pf_hyps : goal sigma -> var_context -(*val pf_untyped_hyps : goal sigma -> (identifier * constr) list*) +(*i val pf_untyped_hyps : goal sigma -> (identifier * constr) list i*) val pf_hyps_types : goal sigma -> (identifier * constr) list val pf_nth_hyp_id : goal sigma -> int -> identifier val pf_last_hyp : goal sigma -> var_declaration |
