aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool/Sumbool.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-23 21:51:50 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-23 21:51:50 +0000
commitac455c1a9fc24c79903251974cbe84e19cb392f4 (patch)
treed9ab38267a064bd3d4985467a3d9b92f14f016e0 /theories/Bool/Sumbool.v
parent123817e082cea45d26b13461caa39807c38ed8a6 (diff)
Remplacement de Induction/Destruct par NewInduction/NewDestruct
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4465 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool/Sumbool.v')
-rw-r--r--theories/Bool/Sumbool.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Bool/Sumbool.v b/theories/Bool/Sumbool.v
index 052df55b1..779969e6f 100644
--- a/theories/Bool/Sumbool.v
+++ b/theories/Bool/Sumbool.v
@@ -17,19 +17,19 @@
Definition sumbool_of_bool : (b:bool) {b=true}+{b=false}.
Proof.
- Induction b; Auto.
+ NewDestruct b; Auto.
Defined.
Hints Resolve sumbool_of_bool : bool.
Definition bool_eq_rec : (b:bool)(P:bool->Set)
((b=true)->(P true))->((b=false)->(P false))->(P b).
-Induction b; Auto.
+NewDestruct b; Auto.
Defined.
Definition bool_eq_ind : (b:bool)(P:bool->Prop)
((b=true)->(P true))->((b=false)->(P false))->(P b).
-Induction b; Auto.
+NewDestruct b; Auto.
Defined.