aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-12 15:58:10 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-12 15:58:10 +0000
commitf7967b6c3e03dabe71cf38d51557b4d94253ae75 (patch)
tree9ed211a781099225bd8fc63e93a39172f34b0a1f /proofs
parentc553366ec1cc485f6ec791ae1c04bbc53f5c65d0 (diff)
Hint Unfold Local + commentaires
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1088 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
-rw-r--r--proofs/pfedit.ml4
-rw-r--r--proofs/refiner.ml26
2 files changed, 16 insertions, 14 deletions
diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml
index 0426955bc..df0c493d5 100644
--- a/proofs/pfedit.ml
+++ b/proofs/pfedit.ml
@@ -58,7 +58,7 @@ let get_state () =
let get_topstate () = snd(get_state())
let get_pftreestate () = fst(get_state())
-(*
+(*i
let get_evmap_sign og =
let og = match og with
| Some n ->
@@ -74,7 +74,7 @@ let get_evmap_sign og =
match og with
| Some goal -> (project goal, pf_env goal)
| _ -> (Evd.empty, Global.env())
-*)
+i*)
let get_goal_context n =
let pftree = get_pftreestate () in
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 840d24b41..4a44a5d14 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -61,10 +61,11 @@ let rec norm_evar_pf sigma p =
ref = Some(r, List.map (norm_evar_pf sigma) pfl)}
-(* mapshape [ l1 ; ... ; lk ] [ v1 ; ... ; vk ] [ p_1 ; .... ; p_(l1+...+lk) ]
+(* [mapshape [ l1 ; ... ; lk ] [ v1 ; ... ; vk ] [ p_1 ; .... ; p_(l1+...+lk) ]]
gives
[ (v1 [p_1 ... p_l1]) ; (v2 [ p_(l1+1) ... p_(l1+l2) ]) ; ... ;
- (vk [ p_(l1+...+l(k-1)+1) ... p_(l1+...lk) ]) ] *)
+ (vk [ p_(l1+...+l(k-1)+1) ... p_(l1+...lk) ]) ]
+ *)
let rec mapshape nl (fl : (proof_tree list -> proof_tree) list)
(l : proof_tree list) =
@@ -74,9 +75,10 @@ let rec mapshape nl (fl : (proof_tree list -> proof_tree) list)
let m,l = list_chop h l in
(List.hd fl m) :: (mapshape t (List.tl fl) l)
-(* frontier : proof_tree -> goal list * validation
- given a proof p, frontier p gives (l,v) where l is the list of goals
- to be solved to complete the proof, and v is the corresponding validation *)
+(* [frontier : proof_tree -> goal list * validation]
+ given a proof [p], [frontier p] gives [(l,v)] where [l] is the list of goals
+ to be solved to complete the proof, and [v] is the corresponding
+ validation *)
let rec frontier p =
match p.ref with
@@ -99,8 +101,8 @@ let rec frontier p =
goal = p.goal;
ref = Some(r,pfl')}))
-(* list_pf p is the lists of goals to be solved in order to complete the
- proof p *)
+(* [list_pf p] is the lists of goals to be solved in order to complete the
+ proof [p] *)
let list_pf p = fst (frontier p)
@@ -212,16 +214,16 @@ let refiner = function
let context ctxt = refiner (Context ctxt)
let vernac_tactic texp = refiner (Tactic texp)
-(* rc_of_pfsigma : proof sigma -> readable_constraints *)
+(* [rc_of_pfsigma : proof sigma -> readable_constraints] *)
let rc_of_pfsigma sigma = rc_of_gc sigma.sigma sigma.it.goal
-(* rc_of_glsigma : proof sigma -> readable_constraints *)
+(* [rc_of_glsigma : proof sigma -> readable_constraints] *)
let rc_of_glsigma sigma = rc_of_gc sigma.sigma sigma.it
-(* extract_open_proof : proof_tree -> constr * (int * constr) list
+(* [extract_open_proof : proof_tree -> constr * (int * constr) list]
takes a (not necessarly complete) proof and gives a pair (pfterm,obl)
where pfterm is the constr corresponding to the proof
- and obl is an int*constr list [ (m1,c1) ; ... ; (mn,cn)]
+ and [obl] is an [int*constr list] [ (m1,c1) ; ... ; (mn,cn)]
where the mi are metavariables numbers, and ci are their types.
Their proof should be completed in order to complete the initial proof *)
@@ -288,7 +290,7 @@ let idtac_valid = function
| _ -> anomaly "Refiner.idtac_valid"
;;
-(* goal_goal_list : goal sigma -> goal list sigma *)
+(* [goal_goal_list : goal sigma -> goal list sigma] *)
let goal_goal_list gls = {it=[gls.it];sigma=gls.sigma};;
(* the identity tactic *)