aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-21 18:47:18 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-21 18:47:18 +0000
commitb00f8fba2259c027757504b2245a81ca40fbb831 (patch)
tree190016608577bf7e3599766706f7c64f4865df88 /theories/ZArith
parent9fc6e8201ea567a6b2c4ba115ce595791a67d336 (diff)
Adaptation à la nouvelle sémantique plus uniforme de "Match term"
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3567 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/Zsqrt.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/theories/ZArith/Zsqrt.v b/theories/ZArith/Zsqrt.v
index 1a78c90df..1293ec6c2 100644
--- a/theories/ZArith/Zsqrt.v
+++ b/theories/ZArith/Zsqrt.v
@@ -25,17 +25,16 @@ Tactic Definition compute_POS :=
| [|- [(POS (xI ?1))]] -> Let v = ?1 In
(Match v With
| [ [xH] ] ->
- (Fail 1)
+ Fail
|_->
Rewrite (POS_xI v))
| [ |- [(POS (xO ?1))]] -> Let v = ?1 In
Match v With
|[ [xH] ]->
- (Fail 1)
+ Fail
|[?]->
Rewrite (POS_xO v)).
-
Inductive sqrt_data [n : Z] : Set :=
c_sqrt: (s, r :Z)`n=s*s+r`->`0<=r<=2*s`->(sqrt_data n) .