aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-03-15 16:37:07 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-03-15 16:37:07 +0000
commitc09f4b75c1c924098cafe7ef23cdb7871a56692d (patch)
tree2d5efe7c01a5175a379fdd7fc4e61a9369e7092a
parent3636d52354226848ef89fbe4539cfa4e5daaa170 (diff)
Typos
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9708 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--theories/Logic/ClassicalFacts.v12
1 files changed, 8 insertions, 4 deletions
diff --git a/theories/Logic/ClassicalFacts.v b/theories/Logic/ClassicalFacts.v
index 896fddc75..ad9171843 100644
--- a/theories/Logic/ClassicalFacts.v
+++ b/theories/Logic/ClassicalFacts.v
@@ -31,8 +31,8 @@ Table of contents:
3.1. Weak excluded middle
-3.2. Gödel-Dummet axiom and right distributivity of implication over
- disjunction
+3.2. Gödel-Dummett axiom and right distributivity of implication over
+ disjunction
3 3. Independence of general premises and drinker's paradox
@@ -396,7 +396,7 @@ End Proof_irrelevance_CCI.
(** We show the following increasing in the strength of axioms:
- weak excluded-middle
- - right distributivity of implication over disjunction and Gödel-Dummet axiom
+ - right distributivity of implication over disjunction and Gödel-Dummett axiom
- independence of general premises and drinker's paradox
- excluded-middle
*)
@@ -533,7 +533,11 @@ Proof.
Qed.
(** Independence of general premises is weaker than (generalized)
- excluded middle *)
+ excluded middle
+
+Remark: generalized excluded middle is preferred here to avoid relying on
+the "ex falso quodlibet" property (i.e. [False -> forall A, A])
+*)
Definition generalized_excluded_middle :=
forall A B:Prop, A \/ (A -> B).