aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-07 17:49:39 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-07 17:49:39 +0000
commit6faf00341b4bcf11884c46c0ab15a2e30265d3e3 (patch)
tree46c4e0e3fc9bb2bd2f74c09a14a9bda369afaf38 /theories7
parent64bf0485dc98d00782ea8d348eef9ea9c6352a11 (diff)
Vieille syntaxe
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5183 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rwxr-xr-xtheories7/Init/Logic.v11
1 files changed, 5 insertions, 6 deletions
diff --git a/theories7/Init/Logic.v b/theories7/Init/Logic.v
index 318b588a8..84a545f3f 100755
--- a/theories7/Init/Logic.v
+++ b/theories7/Init/Logic.v
@@ -101,18 +101,17 @@ Notation "'IF' c1 'then' c2 'else' c3" := (IF c1 c2 c3)
(** First-order quantifiers *)
- (** [(ex A P)], or simply [(EX x | P(x))], expresses the existence of an
+ (** [ex A P], or simply [exists x, P x], expresses the existence of an
[x] of type [A] which satisfies the predicate [P] ([A] is of type
[Set]). This is existential quantification. *)
- (** [(ex2 A P Q)], or simply [(EX x | P(x) & Q(x))], expresses the
+ (** [ex2 A P Q], or simply [exists2 x, P x & Q x], expresses the
existence of an [x] of type [A] which satisfies both the predicates
[P] and [Q] *)
(** Universal quantification (especially first-order one) is normally
- written [(x:A)(P x)]. For duality with existential quantification, the
- construction [(all A P)], or simply [(All P)], is provided as an
- abbreviation of [(x:A)(P x)] *)
+ written [forall x:A, P x]. For duality with existential quantification,
+ the construction [all P] is provided too *)
Inductive ex [A:Type;P:A->Prop] : Prop
:= ex_intro : (x:A)(P x)->(ex A P).
@@ -173,7 +172,7 @@ Section universal_quantification.
(** Equality *)
-(** [(eq A x y)], or simply [x=y], expresses the (Leibniz') equality
+(** [eq A x y], or simply [x=y], expresses the (Leibniz') equality
of [x] and [y]. Both [x] and [y] must belong to the same type [A].
The definition is inductive and states the reflexivity of the equality.
The others properties (symmetry, transitivity, replacement of