aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/ClassicalFacts.v
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 /theories/Logic/ClassicalFacts.v
parente964da1ad108e2bc1f5f01f4ad041c10a07f5d6f (diff)
Commentaires
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5512 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/ClassicalFacts.v')
-rw-r--r--theories/Logic/ClassicalFacts.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Logic/ClassicalFacts.v b/theories/Logic/ClassicalFacts.v
index aa4960a35..8e1696f87 100644
--- a/theories/Logic/ClassicalFacts.v
+++ b/theories/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 := forall A:Prop, A = True \/ A = False.
(** [prop_extensionality] asserts equivalent formulas are equal *)
@@ -216,4 +216,4 @@ End Proof_irrelevance_CIC.
satisfy propositional degeneracy without satisfying proof-irrelevance
(nor dependent case analysis). This would imply that the previous
results cannot be refined.
-*) \ No newline at end of file
+*)