]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library_auto/auto/nat/relevant_equations.ma
auto and autogui... some work
[helm.git] / helm / software / matita / library_auto / auto / nat / relevant_equations.ma
index e057351b36f048ab6dafc6a0bb46cd25689b38d8..8dee78c4fd7e02fa394e28c63c4ef8754aee6fd2 100644 (file)
@@ -12,7 +12,7 @@
 (*                                                                        *)
 (**************************************************************************)
 
-set "baseuri" "cic:/matita/library_auto/nat/relevant_equations".
+set "baseuri" "cic:/matita/library_autobatch/nat/relevant_equations".
 
 include "auto/nat/times.ma".
 include "auto/nat/minus.ma".
@@ -23,7 +23,7 @@ theorem times_plus_l: \forall n,m,p:nat. (n+m)*p = n*p + m*p.
 intros.
 apply (trans_eq ? ? (p*(n+m)))
 [ apply sym_times
-| apply (trans_eq ? ? (p*n+p*m));auto
+| apply (trans_eq ? ? (p*n+p*m));autobatch
   (*[ apply distr_times_plus
   | apply eq_f2;
       apply sym_times    
@@ -35,7 +35,7 @@ theorem times_minus_l: \forall n,m,p:nat. (n-m)*p = n*p - m*p.
 intros.
 apply (trans_eq ? ? (p*(n-m)))
 [ apply sym_times
-| apply (trans_eq ? ? (p*n-p*m));auto
+| apply (trans_eq ? ? (p*n-p*m));autobatch
   (*[ apply distr_times_minus
   | apply eq_f2;
       apply sym_times
@@ -46,7 +46,7 @@ qed.
 theorem times_plus_plus: \forall n,m,p,q:nat. (n + m)*(p + q) =
 n*p + n*q + m*p + m*q.
 intros.
-auto.
+autobatch.
 (*apply (trans_eq nat ? ((n*(p+q) + m*(p+q))))
 [ apply times_plus_l
 | rewrite > distr_times_plus.