From: Andrea Asperti Date: Thu, 23 Nov 2006 13:56:30 +0000 (+0000) Subject: Fixed a call to auto, and commented the remaining part. X-Git-Tag: make_still_working~6652 X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=commitdiff_plain;h=a45b20401c52a767eb8fef71a72be6dc5db8a02a;p=helm.git Fixed a call to auto, and commented the remaining part. --- diff --git a/helm/software/matita/library/technicalities/setoids.ma b/helm/software/matita/library/technicalities/setoids.ma index 4d23d7725..5c19f925e 100644 --- a/helm/software/matita/library/technicalities/setoids.ma +++ b/helm/software/matita/library/technicalities/setoids.ma @@ -246,10 +246,11 @@ definition equality_morphism_of_symmetric_reflexive_transitive_relation: intro; unfold transitive in H; unfold symmetric in sym; - auto. + auto depth=4. ] qed. +(* definition equality_morphism_of_asymmetric_areflexive_transitive_relation: ∀(A: Type)(Aeq: relation A)(trans: transitive ? Aeq). let ASetoidClass1 := AsymmetricAreflexive Contravariant Aeq in @@ -257,7 +258,7 @@ definition equality_morphism_of_asymmetric_areflexive_transitive_relation: (Morphism_Theory (cons ASetoidClass1 (singl ASetoidClass2)) Impl_Relation_Class). intros. exists Aeq. - unfold make_compatibility_goal; simpl; unfold impl; eauto. + unfold make_compatibility_goal; simpl; unfold impl; auto. qed. definition equality_morphism_of_asymmetric_reflexive_transitive_relation: @@ -745,3 +746,4 @@ Ltac refl_st := match goal with definition gen_st : ∀A : Set. Setoid_Theory ? (@eq A). Proof. constructor; congruence. Qed. +*) \ No newline at end of file