如何利用Coq中含有forall的假设?

时间:2017-07-06 07:41:34

标签: coq coq-tactic

我试图在排除中间的假设下证明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,包括使用战术leftright,如果我的证据到现在为止有意义。

提前感谢任何建议和建议!

1 个答案:

答案 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.