aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/ListSet.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-20 16:46:15 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-20 16:46:15 +0000
commitb6337996e891f3fa33e0ff01a7dae13c469d6055 (patch)
tree119d52ec97de7ad8e56d9b5c74373e3a4fd5a954 /theories/Lists/ListSet.v
parentf8a0d5e7f5efcd588627a2eadeb6e8f9f7d597c6 (diff)
portage Refine
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@559 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/ListSet.v')
-rw-r--r--theories/Lists/ListSet.v16
1 files changed, 10 insertions, 6 deletions
diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v
index 6de241d18..a1c86e78f 100644
--- a/theories/Lists/ListSet.v
+++ b/theories/Lists/ListSet.v
@@ -7,14 +7,14 @@
(* PolyList is loaded, but not exported *)
(* This allow to "hide" the definitions, functions and theorems of PolyList
- and to see only the ones of ListSet *)
+ and to see only the ones of ListSet *)
+
Require PolyList.
Implicit Arguments On.
Section first_definitions.
-
Variable A : Set.
Hypothesis Aeq_dec : (x,y:A){x=y}+{~x=y}.
@@ -87,10 +87,14 @@ Section first_definitions.
Proof.
Unfold set_In.
- Realizer set_mem.
- Program_all.
- Rewrite e; Simpl; Auto with datatypes.
- Simpl; Unfold not; Intros [Hc1 | Hc2 ]; Auto with datatypes.
+ (*** Realizer set_mem. Program_all. ***)
+ Induction x.
+ Auto.
+ Intros a0 x0 Ha0. Case (Aeq_dec a a0); Intro eq.
+ Rewrite eq; Simpl; Auto with datatypes.
+ Elim Ha0.
+ Auto with datatypes.
+ Right; Simpl; Unfold not; Intros [Hc1 | Hc2 ]; Auto with datatypes.
Save.
Lemma set_mem_ind :