I'm having trouble with some pretty simple proofs in Coq, using the MathComp library for reflection.
Suppose I want to prove this Lemma:
From mathcomp Require Import ssreflect ssrbool ssrnat.
Lemma example m n: n.+1 < m -> n < m.
Proof.
have predn_ltn_k k: (0 < k.-1) -> (0 < k).
by case: k.
rewrite -subn_gt0 subnS => submn_pred_gt0.
by rewrite -subn_gt0; apply predn_ltn_k.
Qed.
This approach seems a little "unorthodox" to me for such a simple task. Is there a better/simpler way to do this?