我试图在排除中间的假设下证明P \/ Q
和~ P -> Q
的等价性,
Theorem eq_of_or :
excluded_middle ->
forall P Q : Prop,
(P \/ Q) <-> (~ P -> Q).
排除中间区域如下。
Definition excluded_middle := forall P : Prop, P \/ ~ P.
实际上,一个方向的证明不需要排除中间。在我试图证明另一个方向时,当我试图在假设中利用排除中间时,我陷入困境,
Proof.
intros EM P Q. split.
{ intros [H | H]. intros HNP.
- unfold not in HNP. exfalso.
apply HNP. apply H.
- intros HNP. apply H. }
{ intros H. unfold excluded_middle in EM.
unfold not in EM. unfold not in H.
}
当前环境如下:
1 subgoal
EM : forall P : Prop, P \/ (P -> False)
P, Q : Prop
H : (P -> False) -> Q
______________________________________(1/1)
P \/ Q
据我所知,在这种情况下,我们接下来需要做的是做一些类似于&#34;案例分析&#34; P,包括使用战术left
和right
,如果我的证据到现在为止有意义。
提前感谢任何建议和建议!
答案 0 :(得分:2)
你可以用任何命题实例化EM : forall P : Prop, P \/ ~ P
(我用下面的P
实例化它并立即破坏它),因为
EM
本质上是一个采用任意命题P
的函数,并返回P
或~ P
的证据。
Theorem eq_of_or' :
excluded_middle ->
forall P Q : Prop, (~ P -> Q) -> P \/ Q.
Proof.
intros EM P Q.
destruct (EM P) as [p | np]. (* <- the key part is here *)
- left. apply p.
- right.
apply (H np).
(* or, equivalently, *)
Undo.
apply H.
apply np.
Undo 2.
(* we can also combine two `apply` into one: *)
apply H, np.
Qed.