aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/ConstructiveEpsilon.v
diff options
context:
space:
mode:
authorGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-01-23 22:08:35 +0000
committerGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-01-23 22:08:35 +0000
commit9b2ebb8556e6804f5c7490f0a63350487652fc73 (patch)
treed806761a0b1f72e508eccab242d773f052d2f7bc /theories/Logic/ConstructiveEpsilon.v
parentd1bad938698f9998aa66556ac7ed63fb9557754d (diff)
Changing R to a local definition so that it isn't exported.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10470 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/ConstructiveEpsilon.v')
-rw-r--r--theories/Logic/ConstructiveEpsilon.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Logic/ConstructiveEpsilon.v b/theories/Logic/ConstructiveEpsilon.v
index 98260c7fc..36ff2681b 100644
--- a/theories/Logic/ConstructiveEpsilon.v
+++ b/theories/Logic/ConstructiveEpsilon.v
@@ -49,7 +49,7 @@ numbers we try. Namely, [y] is [R]-less then [x] if we try [y] after
infinite [R]-descending chain from 0 is equivalent to the termination
of our searching algorithm. *)
-Definition R (x y : nat) : Prop := x = S y /\ ~ P y.
+Let R (x y : nat) : Prop := x = S y /\ ~ P y.
Notation Local "'acc' x" := (Acc R x) (at level 10).