Let me complete Pierre's answer a little. Because it is easy to find this
proof a bit mysterious.
First, excluded middle is `âA:Prop, AâšÂ¬A`. It is evidently at least as
strong as `âA:Prop, ¬¬(AâšÂ¬A)`. And since the latter is provable in Coq,
excluded middle is actually stronger. It is a general principle in
constructive mathematics that adding double-negations in a statement can be
used to make it weaker: an equivalent principle to excluded middle is
double-negation elimination `âA:Prop, ¬¬AâA`, since it doesn't hold in
constructive mathematics, adding double-negation makes it, in general,
easier to prove a statement.
The principle behind the proof of `âA:Prop, ¬¬(AâšÂ¬A)` is as follows.
First remark that `âA:Prop, ¬(Aâ§Â¬A)` is provable. The definition of `¬A`
being "a contradiction can be derived from `A`", it should be reasonably
clear that this property holds in Coq.
The next step is to prove that `âA B:Prop, ¬(AâšB) â ¬Aâ§Â¬B` (in fact it is
an equivalence). This is a de Morgan law which holds even without excluded
middle. It is true because given a proof of `A`, I can build a proof of
`AâšB` which together with `¬(AâšB)` is contradictory, so `¬A` follows from
`¬(AâšB)`. Symmetrically, so does `¬B`.
Now, suppose `¬(AâšÂ¬A)`, by the above property, we have `¬Aâ§Â¬Â¬A`. By the
first remark, we have a contradiction. Qed.
Post by Pierre CasteranHi,
Assuming ~(A \/ ~A), you first prove ~A, then find a contradiction.
Goal forall A:Prop, ~ ~(A \/ ~A).
intros A H.
apply H.
right;intro a.
destruct H;now left.
Qed.
Pierre
Post by shengyu shenI am trying to prove an exercise in coq art ââA: Prop, âŒâŒ(AâšâŒA).â
I think this may need exclude middle rule, which is not in âCalculus of
Inductive Constructionsâ
am I right?
Shen