aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-03-17 00:11:13 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-03-17 00:11:13 +0000
commitad00dde8284e9476f98e7ad1ff90c8c95939a50e (patch)
tree18c4c9dd71915544f6be7b1562dd70f238b8b252 /theories7
parente964da1ad108e2bc1f5f01f4ad041c10a07f5d6f (diff)
Commentaires
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5512 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rw-r--r--theories7/Logic/ClassicalDescription.v2
-rw-r--r--theories7/Logic/ClassicalFacts.v4
2 files changed, 3 insertions, 3 deletions
diff --git a/theories7/Logic/ClassicalDescription.v b/theories7/Logic/ClassicalDescription.v
index ea2f4f727..37611923a 100644
--- a/theories7/Logic/ClassicalDescription.v
+++ b/theories7/Logic/ClassicalDescription.v
@@ -27,7 +27,7 @@ Axiom dependent_description :
((x:A)(EX y:(B x)|(R x y)/\ ((y':(B x))(R x y') -> y=y')))
-> (EX f:(x:A)(B x) | (x:A)(R x (f x))).
-(** Principle of definite description (aka axiom of unique choice) *)
+(** Principle of definite descriptions (aka axiom of unique choice) *)
Theorem description :
(A:Type;B:Type;R: A->B->Prop)
diff --git a/theories7/Logic/ClassicalFacts.v b/theories7/Logic/ClassicalFacts.v
index 622e6959d..f70d886b3 100644
--- a/theories7/Logic/ClassicalFacts.v
+++ b/theories7/Logic/ClassicalFacts.v
@@ -10,8 +10,8 @@
(** Some facts and definitions about classical logic *)
-(** [prop_degeneracy] asserts (up to consistency) that there are only *)
-(* two distinct formulas *)
+(** [prop_degeneracy] (also referred as propositional completeness) *)
+(* asserts (up to consistency) that there are only two distinct formulas *)
Definition prop_degeneracy := (A:Prop) A==True \/ A==False.
(** [prop_extensionality] asserts equivalent formulas are equal *)