Require Import Coq.Logic.JMeq.
Inductive Le : nat -> nat -> Set :=
| LeO : forall n:nat, Le 0 n
| LeS : forall n m:nat, Le n m -> Le (S n) (S m).
Parameter P : nat -> nat -> Prop.
Goal forall n m:nat, Le (S n) m -> P n m.
intros n m H.
generalize_eqs H.