aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-06 13:59:20 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-06 13:59:20 +0000
commit7643d25ed49d3ccc7b4f9a39f243d5eca4a568d2 (patch)
treeba52421ccae34ef4e67e6fa855c4c6a613b6125d /theories
parent2269d0844f8f8bc25bb2517cc90e02ad5c0e67bc (diff)
Quelques Hint inutiles
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9025 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Lists/List.v11
1 files changed, 2 insertions, 9 deletions
diff --git a/theories/Lists/List.v b/theories/Lists/List.v
index ffe3ac533..62fc994f9 100644
--- a/theories/Lists/List.v
+++ b/theories/Lists/List.v
@@ -135,13 +135,11 @@ Section Facts.
Proof.
simpl in |- *; auto.
Qed.
- Hint Resolve in_eq.
Theorem in_cons : forall (a b:A) (l:list A), In b l -> In b (a :: l).
Proof.
simpl in |- *; auto.
Qed.
- Hint Resolve in_cons.
Theorem in_nil : forall a:A, ~ In a nil.
Proof.
@@ -197,8 +195,6 @@ Section Facts.
induction l; simpl in |- *; auto.
rewrite <- IHl; auto.
Qed.
- Hint Resolve app_nil_end.
-
(** [app] is associative *)
Theorem app_ass : forall l m n:list A, (l ++ m) ++ n = l ++ m ++ n.
@@ -211,9 +207,8 @@ Section Facts.
Theorem ass_app : forall l m n:list A, l ++ m ++ n = (l ++ m) ++ n.
Proof.
- auto.
+ auto using app_ass.
Qed.
- Hint Resolve ass_app.
(** [app] commutes with [cons] *)
Theorem app_comm_cons : forall (x y:list A) (a:A), a :: (x ++ y) = (a :: x) ++ y.
@@ -296,7 +291,6 @@ Section Facts.
now_show ((a0 = a \/ In a y) \/ In a m).
elim (H H1); auto.
Qed.
- Hint Immediate in_app_or.
Lemma in_or_app : forall (l m:list A) (a:A), In a l \/ In a m -> In a (l ++ m).
Proof.
@@ -313,7 +307,6 @@ Section Facts.
now_show (H = a \/ In a (y ++ m)).
elim H2; auto.
Qed.
- Hint Resolve in_or_app.
End Facts.
@@ -890,7 +883,7 @@ Section ListOps.
break_list l1 b l1' H0; break_list l3 c l3' H1.
auto.
apply perm_trans with (l3'++c::l4); auto.
- apply perm_trans with (l1'++a::l2); auto.
+ apply perm_trans with (l1'++a::l2); auto using Permutation_cons_app.
apply perm_skip.
apply (IH a l1' l2 l3' l4); auto.
(* swap *)