aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Div2.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-20 19:48:10 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-20 19:48:10 +0000
commitbe670deace370127c44e1ee3583e61ed6492382a (patch)
tree60ee5bbcab90fea8372f28bd2b71e7af1c9c087b /theories/Arith/Div2.v
parent30cc204e35e6ff422396b85d3b649d38f6a97c1e (diff)
OubliƩ de supprimer du code mort
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1171 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Div2.v')
-rw-r--r--theories/Arith/Div2.v7
1 files changed, 0 insertions, 7 deletions
diff --git a/theories/Arith/Div2.v b/theories/Arith/Div2.v
index 202e7a97a..f5e7ebb34 100644
--- a/theories/Arith/Div2.v
+++ b/theories/Arith/Div2.v
@@ -118,13 +118,6 @@ Simpl. Rewrite (double_S (div2 n0)). Intro H. Injection H. Auto with arith.
Intro H. Inversion H. Inversion H1.
Simpl. Rewrite (double_S (div2 n0)). Auto with arith.
Simpl. Rewrite (double_S (div2 n0)). Intro H. Injection H. Auto with arith.
-(*
-Simpl. Rewrite <- plus_n_Sm. Auto with arith.
-Simpl. Rewrite <- plus_n_Sm. Intro H. Injection H. Auto with arith.
-Intro H. Inversion H. Inversion H1.
-Simpl. Rewrite <- plus_n_Sm. Auto with arith.
-Simpl. Rewrite <- plus_n_Sm. Intro H. Injection H. Auto with arith.
-*)
Qed.