]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/nat/bertrand.ma
generalize no more required before elim
[helm.git] / helm / software / matita / library / nat / bertrand.ma
index 7a0363a58117f7455ef7ed127ef339542c151369..17f4c72e0078ded8e054dc4e750e26aa6b876ea5 100644 (file)
@@ -42,10 +42,10 @@ let rec checker l \def
          | cons h2 t2 => (andb (checker t1) (leb h1 (2*h2))) ]].
 
 lemma checker_cons : \forall t,l.checker (t::l) = true \to checker l = true.
-intros 2;simplify;intro;generalize in match H;elim l
+intros 2;simplify;intro;elim l in H ⊢ %
   [reflexivity
-  |change in H2 with (andb (checker (a::l1)) (leb t (a+(a+O))) = true);
-   apply (andb_true_true ? ? H2)]
+  |change in H1 with (andb (checker (a::l1)) (leb t (a+(a+O))) = true);
+   apply (andb_true_true ? ? H1)]
 qed.
 
 theorem checker_sound : \forall l1,l2,l,x,y.l = l1@(x::y::l2) \to