aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Uniset.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-23 21:00:49 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-23 21:00:49 +0000
commit19dd83cf1b0e57fb13a8d970251822afd6a04ced (patch)
tree7f5630f3f9a54d06f48ad5a1da6d2987332cc01b /theories/Sets/Uniset.v
parent8a95a21a90188d8ef4bd790563a63fdf9b4318a9 (diff)
Remplacement de Induction/Destruct par NewInduction/NewDestruct
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4463 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sets/Uniset.v')
-rw-r--r--theories/Sets/Uniset.v16
1 files changed, 8 insertions, 8 deletions
diff --git a/theories/Sets/Uniset.v b/theories/Sets/Uniset.v
index 17b10ae3a..5b28d6c2b 100644
--- a/theories/Sets/Uniset.v
+++ b/theories/Sets/Uniset.v
@@ -54,7 +54,7 @@ Hints Unfold seq.
Lemma leb_refl : (b:bool)(leb b b).
Proof.
-Induction b; Simpl; Auto.
+NewDestruct b; Simpl; Auto.
Qed.
Hints Resolve leb_refl.
@@ -70,21 +70,21 @@ Qed.
Lemma seq_refl : (x:uniset)(seq x x).
Proof.
-Induction x; Unfold seq; Auto.
+NewDestruct x; Unfold seq; Auto.
Qed.
Hints Resolve seq_refl.
Lemma seq_trans : (x,y,z:uniset)(seq x y)->(seq y z)->(seq x z).
Proof.
Unfold seq.
-Induction x; Induction y; Induction z; Simpl; Intros.
+NewDestruct x; NewDestruct y; NewDestruct z; Simpl; Intros.
Rewrite H; Auto.
Qed.
Lemma seq_sym : (x,y:uniset)(seq x y)->(seq y x).
Proof.
Unfold seq.
-Induction x; Induction y; Simpl; Auto.
+NewDestruct x; NewDestruct y; Simpl; Auto.
Qed.
(** uniset union *)
@@ -109,7 +109,7 @@ Hints Resolve union_empty_right.
Lemma union_comm : (x,y:uniset)(seq (union x y) (union y x)).
Proof.
Unfold seq; Unfold charac; Unfold union.
-Induction x; Induction y; Auto with bool.
+NewDestruct x; NewDestruct y; Auto with bool.
Qed.
Hints Resolve union_comm.
@@ -117,14 +117,14 @@ Lemma union_ass :
(x,y,z:uniset)(seq (union (union x y) z) (union x (union y z))).
Proof.
Unfold seq; Unfold union; Unfold charac.
-Induction x; Induction y; Induction z; Auto with bool.
+NewDestruct x; NewDestruct y; NewDestruct z; Auto with bool.
Qed.
Hints Resolve union_ass.
Lemma seq_left : (x,y,z:uniset)(seq x y)->(seq (union x z) (union y z)).
Proof.
Unfold seq; Unfold union; Unfold charac.
-Induction x; Induction y; Induction z.
+NewDestruct x; NewDestruct y; NewDestruct z.
Intros; Elim H; Auto.
Qed.
Hints Resolve seq_left.
@@ -132,7 +132,7 @@ Hints Resolve seq_left.
Lemma seq_right : (x,y,z:uniset)(seq x y)->(seq (union z x) (union z y)).
Proof.
Unfold seq; Unfold union; Unfold charac.
-Induction x; Induction y; Induction z.
+NewDestruct x; NewDestruct y; NewDestruct z.
Intros; Elim H; Auto.
Qed.
Hints Resolve seq_right.