src/Provers/Arith/assoc_fold.ML
author kleing
Tue, 13 May 2003 08:59:21 +0200
changeset 14024 213dcc39358f
parent 13480 bb72bd43c6c3
child 14387 e96d5c42c4b0
permissions -rw-r--r--
HOL-Real -> HOL-Complex
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     1
(*  Title:      Provers/Arith/assoc_fold.ML
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     2
    ID:         $Id$
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     4
    Copyright   1999  University of Cambridge
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     5
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     6
Simplification procedure for associative operators + and * on numeric types
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     7
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     8
Performs constant folding when the literals are separated, as in 3+n+4.
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
     9
*)
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    10
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    11
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    12
signature ASSOC_FOLD_DATA =
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    13
sig
13462
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    14
  val ss                : simpset       (*basic simpset of object-logtic*)
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    15
  val eq_reflection     : thm           (*object-equality to meta-equality*)
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    16
  val sg_ref            : Sign.sg_ref   (*the operator's signature*)
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    17
  val T                 : typ           (*the operator's numeric type*)
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    18
  val plus              : term          (*the operator being folded*)
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    19
  val add_ac            : thm list      (*AC-rewrites for plus*)
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    20
end;
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    21
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    22
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    23
functor Assoc_Fold (Data: ASSOC_FOLD_DATA) =
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    24
struct
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    25
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    26
 val assoc_ss = Data.ss addsimps Data.add_ac;
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    27
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    28
 exception Assoc_fail;
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    29
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    30
 fun mk_sum []  = raise Assoc_fail
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    31
   | mk_sum tms = foldr1 (fn (x,y) => Data.plus $ x $ y) tms;
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    32
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    33
 (*Separate the literals from the other terms being combined*)
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    34
 fun sift_terms (t, (lits,others)) =
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    35
     case t of
13462
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    36
          Const("Numeral.number_of", _) $ _ =>
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    37
              (t::lits, others)         (*new literal*)
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    38
        | (f as Const _) $ x $ y =>
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    39
              if f = Data.plus
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    40
              then sift_terms (x, sift_terms (y, (lits,others)))
13462
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    41
              else (lits, t::others)    (*arbitrary summand*)
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    42
        | _ => (lits, t::others);
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    43
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    44
 val trace = ref false;
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    45
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    46
 (*Make a simproc to combine all literals in a associative nest*)
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    47
 fun proc sg _ lhs =
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    48
   let fun show t = string_of_cterm (Thm.cterm_of sg t)
12262
11ff5f47df6e use tracing function for trace output;
wenzelm
parents: 9419
diff changeset
    49
       val _ = if !trace then tracing ("assoc_fold simproc: LHS = " ^ show lhs)
13462
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    50
               else ()
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    51
       val (lits,others) = sift_terms (lhs, ([],[]))
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    52
       val _ = if length lits < 2
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    53
               then raise Assoc_fail (*we can't reduce the number of terms*)
13462
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    54
               else ()
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    55
       val rhs = Data.plus $ mk_sum lits $ mk_sum others
12262
11ff5f47df6e use tracing function for trace output;
wenzelm
parents: 9419
diff changeset
    56
       val _ = if !trace then tracing ("RHS = " ^ show rhs) else ()
13480
bb72bd43c6c3 use Tactic.prove instead of prove_goalw_cterm in internal proofs!
wenzelm
parents: 13462
diff changeset
    57
       val th = Tactic.prove sg [] [] (Logic.mk_equals (lhs, rhs))
bb72bd43c6c3 use Tactic.prove instead of prove_goalw_cterm in internal proofs!
wenzelm
parents: 13462
diff changeset
    58
                   (fn _ => rtac Data.eq_reflection 1 THEN
bb72bd43c6c3 use Tactic.prove instead of prove_goalw_cterm in internal proofs!
wenzelm
parents: 13462
diff changeset
    59
                            simp_tac assoc_ss 1)
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    60
   in Some th end
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    61
   handle Assoc_fail => None;
13462
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    62
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    63
 val conv =
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    64
     Simplifier.simproc_i (Sign.deref Data.sg_ref) "assoc_fold"
56610e2ba220 sane interface for simprocs;
wenzelm
parents: 12262
diff changeset
    65
       [Data.plus $ Free ("x", Data.T) $ Free ("y",Data.T)] proc;
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    66
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    67
end;
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    68
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    69
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    70
(*test data:
8999
ad8260dc6e4a global timing flag;
wenzelm
parents: 8857
diff changeset
    71
set timing;
7072
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    72
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    73
Goal "(#3 * (a * #34)) * (#2 * b * #9) = (x::int)";
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    74
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    75
Goal "a + b + c + d + e + f + g + h + i + j + k + l + m + n + oo + p + q + r + s + t + u + v + (w + x + y + z + a + #2 + b + #2 + c + #2 + d + #2 + e) + #2 + f + (#2 + g + #2 + h + #2 + i) + #2 + (j + #2 + k + #2 + l + #2 + m + #2) + n + #2 + (oo + #2 + p + #2 + q + #2 + r) + #2 + s + #2 + t + #2 + u + #2 + v + #2 + w + #2 + x + #2 + y + #2 + z + #2 = (uu::nat)";
c3f3fd86e11c new simprocs assoc_fold and combine_coeff
paulson
parents:
diff changeset
    76
*)