aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-02-07 16:51:44 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-02-07 16:51:44 +0000
commit5e8634d9ad5f87404e59f59888b318ca8367afc1 (patch)
tree2fd849398a117e3f41bb606ab3a2764134c411e3 /proofs
parent139f62dc00ad5afc1d81404930b302234e486264 (diff)
Typo in comments.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14972 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
-rw-r--r--proofs/proof.ml4
-rw-r--r--proofs/proof.mli2
2 files changed, 3 insertions, 3 deletions
diff --git a/proofs/proof.ml b/proofs/proof.ml
index 72730495d..748792744 100644
--- a/proofs/proof.ml
+++ b/proofs/proof.ml
@@ -68,8 +68,8 @@ module Cond = struct
(* first attempt at an algebra of condition *)
(* semantics:
- [Cannot] means that the condition is not met
- - [Strict] that the condition is meant
- - [Loose] that the condition is not quite meant
+ - [Strict] that the condition is met
+ - [Loose] that the condition is not quite met
but authorises to unfocus provided a condition
of a previous focus on the stack is (strictly)
met.
diff --git a/proofs/proof.mli b/proofs/proof.mli
index 12af18f40..7c538cf0e 100644
--- a/proofs/proof.mli
+++ b/proofs/proof.mli
@@ -151,7 +151,7 @@ val run_tactic : Environ.env -> unit Proofview.tactic -> proof -> unit
a focusing command and a tactic. Transactions are such that if
any of the atomic action fails, the whole transaction fails.
- During a transaction, the undo visible undo stack is constituted only
+ During a transaction, the visible undo stack is constituted only
of the actions performed done during the transaction.
[transaction p f] can be called on an [f] using, itself, [transaction p].*)