aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar thery <thery@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-19 09:21:52 +0000
committerGravatar thery <thery@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-19 09:21:52 +0000
commitbdb10644ba3f905e274c98b73a5ba35d121b6a37 (patch)
tree57db293e3c2f0899d601e9f3f406966a11c10943 /theories
parentae4c0218bb7544a0791620e83024fcc930606bba (diff)
genN.ml sync
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9893 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Ints/num/genN.ml18
1 files changed, 11 insertions, 7 deletions
diff --git a/theories/Ints/num/genN.ml b/theories/Ints/num/genN.ml
index 775237f6a..43e771972 100644
--- a/theories/Ints/num/genN.ml
+++ b/theories/Ints/num/genN.ml
@@ -1,6 +1,6 @@
open Format
-let size = 3
+let size = 12
let sizeaux = 1
let t = "t"
@@ -12,7 +12,7 @@ let basename = "N"
let print_header fmt l =
let l = "ZArith"::"Basic_type"::"ZnZ"::"Zn2Z"::"Nbasic"::"GenMul"::
- "GenDivn1"::"Lucas"::l in
+ "GenDivn1"::l in
List.iter (fun s -> fprintf fmt "Require Import %s.\n" s) l;
fprintf fmt "\n"
@@ -590,9 +590,10 @@ let print_Make () =
for i = 0 to size do
fprintf fmt " Definition w%i_divn1 :=\n" i;
- fprintf fmt " gen_divn1 w%i_op.(znz_digits) w%i_op.(znz_0)\n" i i;
+ fprintf fmt " gen_divn1 w%i_op.(znz_zdigits) w%i_op.(znz_0)\n" i i;
fprintf fmt " w%i_op.(znz_WW) w%i_op.(znz_head0)\n" i i;
- fprintf fmt " w%i_op.(znz_add_mul_div) w%i_op.(znz_div21).\n" i i
+ fprintf fmt " w%i_op.(znz_add_mul_div) w%i_op.(znz_div21)\n" i i;
+ fprintf fmt " w%i_op.(znz_compare) w%i_op.(znz_sub).\n" i i;
done;
fprintf fmt "\n";
@@ -665,10 +666,13 @@ let print_Make () =
for i = 0 to size do
fprintf fmt " Definition w%i_modn1 :=\n" i;
- fprintf fmt " gen_modn1 w%i_op.(znz_digits) w%i_op.(znz_0)\n" i i;
+ fprintf fmt " gen_modn1 w%i_op.(znz_zdigits) w%i_op.(znz_0)\n" i i;
fprintf fmt
- " w%i_op.(znz_head0) w%i_op.(znz_add_mul_div) w%i_op.(znz_div21).\n"
- i i i
+ " w%i_op.(znz_head0) w%i_op.(znz_add_mul_div) w%i_op.(znz_div21)\n"
+ i i i;
+ fprintf fmt
+ " w%i_op.(znz_compare) w%i_op.(znz_sub).\n"
+ i i;
done;
fprintf fmt "\n";