G4iSLt.strong_inductionT

Require Import PeanoNat.

(* Strong induction on Natural numbers with properties sending to Type. *)

Theorem strong_inductionT:
P : Type,
( n : , ( k : , (k < n P k)) P n)
n : , P n.
Proof.
intros P H. assert (Lem : n, ( m, m n P m)).
{ induction n. intros.
  - assert (E: m = 0). inversion . reflexivity. rewrite E. apply H.
    intros. exfalso. inversion .
  - intros. apply H. intros. apply IHn. inversion .
    * rewrite in . apply Nat.lt_succ_r. apply .
    * assert (E: k m). apply Nat.lt_le_incl. apply .
      apply Nat.le_trans with (m:=m). apply E. apply . }
intro n. apply H. intros. apply Lem with (n:=n) (m:=k).
apply Nat.lt_le_incl. apply .
Qed.