From a55947f409f9ea0cb707c72cd5005726eebd33e5 Mon Sep 17 00:00:00 2001 From: msozeau Date: Tue, 31 Jan 2012 16:43:56 +0000 Subject: Revert "Tentative to fix bug #2628 by not letting intuition break records. Might be too much of a backwards-incompatible change" Indeed it is breaking too many scripts. This reverts commit 47e9afaaa4c08aca97d4f4b5a89cb40da76bd850. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14956 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Classes/Equivalence.v | 11 +---------- theories/Classes/Morphisms.v | 7 ------- 2 files changed, 1 insertion(+), 17 deletions(-) (limited to 'theories/Classes') diff --git a/theories/Classes/Equivalence.v b/theories/Classes/Equivalence.v index 87316cda9..d9e9fe257 100644 --- a/theories/Classes/Equivalence.v +++ b/theories/Classes/Equivalence.v @@ -113,12 +113,6 @@ Section Respecting. Solve Obligations using unfold respecting in * ; simpl_relation ; program_simpl. - Next Obligation. - Proof. - unfold respecting in *. program_simpl. transitivity (y y0); auto. symmetry; apply H. reflexivity. - Qed. - - Next Obligation. Proof. unfold respecting in *. program_simpl. transitivity (y y0); auto. apply H0. reflexivity. @@ -128,13 +122,10 @@ End Respecting. (** The default equivalence on function spaces, with higher-priority than [eq]. *) -Hint Extern 0 => reflexivity : relations. -Hint Extern 1 => solve [symmetry; auto] : relations. - Program Instance pointwise_equivalence {A} `(eqb : Equivalence B eqB) : Equivalence (pointwise_relation A eqB) | 9. Next Obligation. Proof. - transitivity (y a); auto with relations. + transitivity (y a) ; auto. Qed. diff --git a/theories/Classes/Morphisms.v b/theories/Classes/Morphisms.v index 30d82822a..8e491b1b8 100644 --- a/theories/Classes/Morphisms.v +++ b/theories/Classes/Morphisms.v @@ -143,13 +143,6 @@ Typeclasses Opaque respectful pointwise_relation forall_relation. Program Instance respectful_per `(PER A R, PER B R') : PER (R ==> R'). - Next Obligation. - Proof with auto. - assert(R x0 x0). - transitivity y0... symmetry... - symmetry... apply H1. now symmetry. - Qed. - Next Obligation. Proof with auto. assert(R x0 x0). -- cgit v1.2.3