While using ssreflect
in the following lemma:
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
Lemma nat_dec n m: (m <= n) -> (~~ (m <= n)) -> False.
Proof.
intros A notA.
(* auto. *)
red in A.
red in notA.
(* auto. *)
rewrite -> A in notA.
auto.
Qed.
May I ask why those autos
, that I commented out, do not work at those proof states? as it seems to me that these states already observe contradiction in the context.
And is there some automation by ssreflect
to prove this lemma?