aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-25 10:19:05 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-25 10:19:05 +0000
commitbe9c3dc93413a76d188724d4a06739d9bb238b72 (patch)
treed59cc88bcf3661ddfcc03ef42902e0d5178f71a8
parent72add906154ce22894a41cf04543a7c096456e09 (diff)
More compatibility fixes, revert the tauto fix that prevented
destruction of records as a lot of scripts currently rely on it. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11263 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--tactics/tauto.ml44
-rw-r--r--theories/Classes/Equivalence.v11
-rw-r--r--theories/Classes/Morphisms.v5
3 files changed, 3 insertions, 17 deletions
diff --git a/tactics/tauto.ml4 b/tactics/tauto.ml4
index 6ce54c5a2..90705c8c9 100644
--- a/tactics/tauto.ml4
+++ b/tactics/tauto.ml4
@@ -56,7 +56,7 @@ let is_binary t =
let is_conj ist =
let ind = assoc_last ist in
- if (is_conjunction ind) && (is_nodep_ind ind) && not (is_record ind)
+ if (is_conjunction ind) && (is_nodep_ind ind) (* && not (is_record ind) *)
&& is_binary ind (* for compatibility, as (?X _ _) matches
applications with 2 or more arguments. *)
then
@@ -65,7 +65,7 @@ let is_conj ist =
<:tactic<fail>>
let is_disj ist =
- if is_disjunction (assoc_last ist) then
+ if is_disjunction (assoc_last ist) && is_binary (assoc_last ist) then
<:tactic<idtac>>
else
<:tactic<fail>>
diff --git a/theories/Classes/Equivalence.v b/theories/Classes/Equivalence.v
index 84aa9cf06..22d9ff56f 100644
--- a/theories/Classes/Equivalence.v
+++ b/theories/Classes/Equivalence.v
@@ -54,9 +54,6 @@ Infix "=~=" := pequiv (at level 70, no associativity) : equiv_scope.
Program Instance equiv_reflexive [ sa : Equivalence A ] : Reflexive equiv.
- Next Obligation.
- Proof. reflexivity. Qed.
-
Program Instance equiv_symmetric [ sa : Equivalence A ] : Symmetric equiv.
Next Obligation.
@@ -127,13 +124,7 @@ Section Respecting.
Next Obligation.
Proof.
- unfold respecting in *. program_simpl. destruct eqa ; destruct eqb. red in H2,H1 ; auto.
- Qed.
-
- Next Obligation.
- Proof.
- unfold respecting in *. program_simpl. destruct eqa ; destruct eqb. red in H2,H3,H4.
- transitivity (y y0) ; auto.
+ unfold respecting in *. program_simpl. transitivity (y y0); auto. apply H0. reflexivity.
Qed.
End Respecting.
diff --git a/theories/Classes/Morphisms.v b/theories/Classes/Morphisms.v
index 0a099e135..8acbe916b 100644
--- a/theories/Classes/Morphisms.v
+++ b/theories/Classes/Morphisms.v
@@ -96,11 +96,6 @@ Program Instance respectful_per [ PER A (R : relation A), PER B (R' : relation B
Next Obligation.
Proof with auto.
- destruct PER0 ; destruct PER1 ; auto.
- Qed.
-
- Next Obligation.
- Proof with auto. destruct PER0 ; destruct PER1.
assert(R x0 x0).
transitivity y0... symmetry...
transitivity (y x0)...