]> matita.cs.unibo.it Git - helm.git/commitdiff
auto => auto new.
authoracciavat <??>
Thu, 12 Oct 2006 09:53:08 +0000 (09:53 +0000)
committeracciavat <??>
Thu, 12 Oct 2006 09:53:08 +0000 (09:53 +0000)
There is still one auto left that does not work with the new implementation
(because of implicative hypothesis for local lemmas?)

helm/software/matita/contribs/CoRN/algebra/Setoids.ma

index 4fcb5a23be061042d8a70235f4dbb6692ced0da5..6b7bf781ddfc429aff3a745393d48bed6b793a1a 100644 (file)
@@ -1227,11 +1227,6 @@ qed.
 
 
 
-axiom proper_caseZ_diff_CS : \forall CS : CSetoid. \forall f : nat \to nat \to CS.
- (\forall m,n,p,q : nat. eq nat (plus m q) (plus n p) \to (f m n) = (f p q)) \to
- \forall m,n : nat. caseZ_diff CS (Zminus (Z_of_nat m) (Z_of_nat n)) f = (f m n).
-
-(*
 lemma proper_caseZ_diff_CS : \forall CS : CSetoid. \forall f : nat \to nat \to CS.
  (\forall m,n,p,q : nat. eq nat (plus m q) (plus n p) \to (f m n) = (f p q)) \to
  \forall m,n : nat. caseZ_diff CS (Zminus (Z_of_nat m) (Z_of_nat n)) f = (f m n).
@@ -1253,9 +1248,9 @@ apply f. apply n1. apply m1.
 apply eq_symmetric_unfolded.assumption.
 apply eq_symmetric_unfolded.assumption.
 apply H.
-auto.
+auto new.
 qed.
-*)
+
 (*
 Finally, we characterize functions defined on the natural numbers also as setoid functions, similarly to what we already did for predicates.
 *)