]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/tests/inversion.ma
auto => auto new everywhere + minor updates to make more tests pass
[helm.git] / helm / software / matita / tests / inversion.ma
index 3e49e06685d22818abd961fec9774f7708b4ab79..35963ab7392bf2b99fba801b6fb3ebf54795fc42 100644 (file)
@@ -42,7 +42,7 @@ theorem t: \forall x,y. \forall H: sum x y O.
  simplify. intros.
  generalize in match H1.
  rewrite < H2; rewrite < H3.intro.
- rewrite > H4.auto.
+ rewrite > H4.auto new.
 qed.
 
 theorem t1: \forall x,y. sum x y O \to x = y.
@@ -57,5 +57,5 @@ apply (sum_ind ? (\lambda a,b,K. y=a \to O=b \to x=a) ? ? ? s).*)
 inversion s.
 intros.simplify.
 intros.
-rewrite > H. rewrite < H2.  auto.
+rewrite > H. rewrite < H2.  auto new.
 qed.