小编Mat*_*chi的帖子

Coq中的双重感应

基本上,我想证明以下结果:

Lemma nat_ind_2 (P: nat -> Prop): P 0 -> P 1 -> (forall n, P n -> P (2+n)) ->
    forall n, P n.
Run Code Online (Sandbox Code Playgroud)

这就是所谓的双重归纳的复发方案.

我试图证明它应用感应两次,但我不确定我会以这种方式得到它.实际上,我在那时陷入困境:

Proof.
  intros. elim n.
    exact H.
    intros. elim n0.
      exact H0.
      intros. apply (H1 n1).
Run Code Online (Sandbox Code Playgroud)

double recurrence coq induction

3
推荐指数
1
解决办法
1077
查看次数

标签 统计

coq ×1

double ×1

induction ×1

recurrence ×1