'0 <a -> 1 <a + 1'的更简单证明

时间:2019-08-01 02:18:30

标签: coq ssreflect

我想知道语句forall a:nat, 0 < a -> 1 < a + 1的简短或更简单的证明。 在mathcomp / ssreflect中。

我有以下证明,但希望有更优雅的证明。

From mathcomp Require Import all_ssreflect.
Goal forall a:nat, 0 < a -> 1 < a + 1.
  move=>a.
  have H:1=0+1 by [].
  by rewrite {2}H ltn_add2r.
Qed.

1 个答案:

答案 0 :(得分:3)

那一个呢?

From mathcomp Require Import all_ssreflect.
Goal forall a:nat, 0 < a -> 1 < a + 1.
by move=>?; rewrite addn1 ltnS.
Qed.