aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/micromega/mutils.ml
diff options
context:
space:
mode:
Diffstat (limited to 'plugins/micromega/mutils.ml')
-rw-r--r--plugins/micromega/mutils.ml17
1 files changed, 0 insertions, 17 deletions
diff --git a/plugins/micromega/mutils.ml b/plugins/micromega/mutils.ml
index 03e3999fd..23db2928a 100644
--- a/plugins/micromega/mutils.ml
+++ b/plugins/micromega/mutils.ml
@@ -14,9 +14,6 @@
let debug = false
-let fst' (Micromega.Pair(x,y)) = x
-let snd' (Micromega.Pair(x,y)) = y
-
let map_option f x =
match x with
| None -> None
@@ -225,11 +222,6 @@ struct
let num x = Num.Big_int (z_big_int x)
- let rec list elt l =
- match l with
- | Nil -> []
- | Cons(e,l) -> (elt e)::(list elt l)
-
let q_to_num {qnum = x ; qden = y} =
Big_int (z_big_int x) // (Big_int (z_big_int (Zpos y)))
@@ -256,10 +248,6 @@ struct
else if nt = 0 then N0
else Npos (positive nt)
-
-
-
-
let rec index n =
if n=1 then XH
else if n land 1 = 1 then XI (index (n lsr 1))
@@ -279,8 +267,6 @@ struct
(List.rev (digits_of_int n))
(XH)
-
-
let z x =
match compare x 0 with
| 0 -> Z0
@@ -311,9 +297,6 @@ struct
{Micromega.qnum = bigint (numerator n) ;
Micromega.qden = positive_big_int (denominator n)}
-
- let list elt l = List.fold_right (fun x l -> Cons(elt x, l)) l Nil
-
end
module Cmp =