]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/arithmetics/nat.ma
This line, and those below, will be ignored--
[helm.git] / matita / matita / lib / arithmetics / nat.ma
index 56935028f65015812b79fdc15fb8762b012d14cf..67b7de50b7dfb5711e9679b502720862e49c6d03 100644 (file)
@@ -495,6 +495,13 @@ cut (∀q:nat. q ≤ n → P q) /2/
  ]
 qed.
 
+lemma f_ind: ∀A. ∀f:A→ℕ. ∀P:predicate A.
+             (∀n. (∀a. f a < n → P a) → ∀a. f a = n → P a) → ∀a. P a.
+#A #f #P #H #a
+cut (∀n,a. f a = n → P a) /2 width=3/ -a
+#n @(nat_elim1 … n) -n #n /3 width=3/ (**) (* auto very slow (274s) without #n *)
+qed-.
+
 (* More negated equalities **************************************************)
 
 theorem lt_to_not_eq : ∀n,m:nat. n < m → n ≠ m.