aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/ListSet.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-02-01 08:35:21 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-02-01 08:35:21 +0000
commitc300bc395fb987f7ded64c17bce5c966c0279442 (patch)
tree443364b05d14feb412ba7a1a66ebc6ee1b6d8b2e /theories/Lists/ListSet.v
parent1fda9cc1a2d8c2db92d88d3e2715d3ee86f90bf3 (diff)
- coqc : option -image
- coqmktop : manquaient des -I - tauto : rétablissement du vieux tauto en attendant la stabilité du nouveau - correction d'un bug de Simpl avec Fix (découvert dans preuve FTA) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1304 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/ListSet.v')
-rw-r--r--theories/Lists/ListSet.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v
index a1c86e78f..3c083aa97 100644
--- a/theories/Lists/ListSet.v
+++ b/theories/Lists/ListSet.v
@@ -189,7 +189,7 @@ Section first_definitions.
Simpl; Intros [H1|H2]; Auto with datatypes.
Simpl; Do 3 Intro.
Elim (Aeq_dec b a0).
- Tauto.
+ Simpl; Tauto.
Simpl; Intros; Elim H0.
Trivial with datatypes.
Tauto.
@@ -271,7 +271,7 @@ Section first_definitions.
(set_In a (set_inter x y)) -> (set_In a y).
Proof.
Induction x.
- Tauto.
+ Simpl; Tauto.
Simpl; Intros a0 l Hrec y.
Generalize (!set_mem_correct1 a0 y).
Elim (set_mem a0 y); Simpl; Intros.
@@ -291,7 +291,7 @@ Section first_definitions.
(set_In a x) -> ~(set_In a y) -> (set_In a (set_diff x y)).
Proof.
Induction x.
- Tauto.
+ Simpl; Tauto.
Simpl; Intros a0 l Hrec y [Ha0a | Hal] Hay.
Rewrite Ha0a; Generalize (set_mem_complete2 Hay).
Elim (set_mem a y); [ Intro Habs; Discriminate Habs | Auto with datatypes ].
@@ -302,7 +302,7 @@ Section first_definitions.
(set_In a (set_diff x y)) -> (set_In a x).
Proof.
Induction x.
- Tauto.
+ Simpl; Tauto.
Simpl; Intros a0 l Hrec y; Elim (set_mem a0 y).
EAuto with datatypes.
Intro; Generalize (set_add_elim H).