aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proofview.ml
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-08-12 11:20:26 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-08-12 11:20:26 +0000
commit02287bddfe994ab4c540599aa4915b6855f94256 (patch)
tree4525411409865c793498b605fac87456f3132ec2 /proofs/proofview.ml
parente44ffa03378eec03425ec8a2698365f95d7dcb81 (diff)
Fixes mini-bug: Qed would succeed even on focused proofs.
It allowed proofs of the Shape [{ solve. Qed.] which is inelegant at best. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14409 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/proofview.ml')
-rw-r--r--proofs/proofview.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/proofs/proofview.ml b/proofs/proofview.ml
index dd65a9049..3964692b1 100644
--- a/proofs/proofview.ml
+++ b/proofs/proofview.ml
@@ -122,7 +122,7 @@ let unfocus_sublist (left,right) s =
(* [focus i j] focuses a proofview on the goals from index [i] to index [j]
(inclusive). (i.e. goals number [i] to [j] become the only goals of the
- returned proofview).
+ returned proofview). The first goal has index 1.
It returns the focus proof, and a context for the focus trace. *)
let focus i j sp =
let (new_comb, context) = focus_sublist i j sp.comb in