]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/nat/factorial2.ma
Prima versione di bertrand. Tanti cambiamenti qua e la.
[helm.git] / helm / software / matita / library / nat / factorial2.ma
index 594feb51f7ec365fe4ea568f9723c2e33d489c13..6215d6657892ab39eb0233763885657f35796725 100644 (file)
@@ -25,11 +25,6 @@ theorem exp_S: \forall n,m. exp m (S n) = m*exp m n.
 intros.reflexivity.
 qed.
 
-alias num (instance 0) = "natural number".
-lemma times_SSO: \forall n.2*(S n) = S(S(2*n)).
-intro.simplify.rewrite < plus_n_Sm.reflexivity.
-qed.
-
 theorem lt_O_to_fact1: \forall n.O<n \to
 fact (2*n) \le (exp 2 (pred (2*n)))*(fact n)*(fact n).
 intros.elim H