src/Provers/Arith/cancel_numerals.ML
author wenzelm
Mon, 01 Aug 2005 19:20:26 +0200
changeset 16973 b2a894562b8f
parent 15965 f422f8283491
child 17223 430edc6b7826
permissions -rw-r--r--
simprocs: Simplifier.inherit_bounds;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
     1
(*  Title:      Provers/Arith/cancel_numerals.ML
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
     2
    ID:         $Id$
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
     4
    Copyright   2000  University of Cambridge
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
     5
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
     6
Cancel common coefficients in balanced expressions:
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
     7
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
     8
     i + #m*u + j ~~ i' + #m'*u + j'  ==  #(m-m')*u + i + j ~~ i' + j'
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
     9
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    10
where ~~ is an appropriate balancing operation (e.g. =, <=, <, -).
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    11
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    12
It works by (a) massaging both sides to bring the selected term to the front:
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    13
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    14
     #m*u + (i + j) ~~ #m'*u + (i' + j') 
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    15
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    16
(b) then using bal_add1 or bal_add2 to reach
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    17
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    18
     #(m-m')*u + i + j ~~ i' + j'       (if m'<=m)
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    19
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    20
or
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    21
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    22
     i + j ~~ #(m'-m)*u + i' + j'       (otherwise)
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    23
*)
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    24
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    25
signature CANCEL_NUMERALS_DATA =
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    26
sig
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    27
  (*abstract syntax*)
14387
e96d5c42c4b0 Polymorphic treatment of binary arithmetic using axclasses
paulson
parents: 13484
diff changeset
    28
  val mk_sum: typ -> term list -> term
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    29
  val dest_sum: term -> term list
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    30
  val mk_bal: term * term -> term
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    31
  val dest_bal: term -> term * term
15965
f422f8283491 Use of IntInf.int instead of int in most numeric simprocs; avoids
paulson
parents: 15570
diff changeset
    32
  val mk_coeff: IntInf.int * term -> term
f422f8283491 Use of IntInf.int instead of int in most numeric simprocs; avoids
paulson
parents: 15570
diff changeset
    33
  val dest_coeff: term -> IntInf.int * term
f422f8283491 Use of IntInf.int instead of int in most numeric simprocs; avoids
paulson
parents: 15570
diff changeset
    34
  val find_first_coeff: term -> term list -> IntInf.int * term list
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    35
  (*rules*)
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    36
  val bal_add1: thm
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    37
  val bal_add2: thm
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    38
  (*proof tools*)
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    39
  val prove_conv: tactic list -> theory -> 
13484
d8f5d3391766 adhoc_freeze_vars;
wenzelm
parents: 9546
diff changeset
    40
                  thm list -> string list -> term * term -> thm option
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    41
  val trans_tac: simpset -> thm option -> tactic (*applies the initial lemma*)
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    42
  val norm_tac: simpset -> tactic                (*proves the initial lemma*)
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    43
  val numeral_simp_tac: simpset -> tactic        (*proves the final theorem*)
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    44
  val simplify_meta_eq: simpset -> thm -> thm    (*simplifies the final theorem*)
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    45
end;
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    46
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    47
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    48
functor CancelNumeralsFun(Data: CANCEL_NUMERALS_DATA):
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    49
  sig
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    50
  val proc: theory -> simpset -> term -> thm option
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    51
  end 
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    52
=
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    53
struct
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    54
8779
2d4afbc46801 various bug fixes
paulson
parents: 8772
diff changeset
    55
(*For t = #n*u then put u in the table*)
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    56
fun update_by_coeff (tab, t) =
8779
2d4afbc46801 various bug fixes
paulson
parents: 8772
diff changeset
    57
  Termtab.update ((#2 (Data.dest_coeff t), ()), tab);
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    58
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    59
(*a left-to-right scan of terms1, seeking a term of the form #n*u, where
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    60
  #m*u is in terms2 for some m*)
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    61
fun find_common (terms1,terms2) =
15570
8d8c70b41bab Move towards standard functions.
skalberg
parents: 15531
diff changeset
    62
  let val tab2 = Library.foldl update_by_coeff (Termtab.empty, terms2)
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    63
      fun seek [] = raise TERM("find_common", []) 
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    64
	| seek (t::terms) =
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    65
	      let val (_,u) = Data.dest_coeff t 
15570
8d8c70b41bab Move towards standard functions.
skalberg
parents: 15531
diff changeset
    66
	      in  if isSome (Termtab.lookup (tab2, u)) then u
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    67
		  else seek terms
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    68
	      end
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    69
  in  seek terms1 end;
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    70
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    71
(*the simplification procedure*)
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    72
fun proc thy ss t =
15027
d23887300b96 adapted type of simprocs;
wenzelm
parents: 14387
diff changeset
    73
  let
d23887300b96 adapted type of simprocs;
wenzelm
parents: 14387
diff changeset
    74
      val hyps = prems_of_ss ss;
d23887300b96 adapted type of simprocs;
wenzelm
parents: 14387
diff changeset
    75
      (*first freeze any Vars in the term to prevent flex-flex problems*)
13484
d8f5d3391766 adhoc_freeze_vars;
wenzelm
parents: 9546
diff changeset
    76
      val (t', xs) = Term.adhoc_freeze_vars t;
9191
300bd596d696 now freezes Vars in order to prevent errors in cases like these:
paulson
parents: 8799
diff changeset
    77
      val (t1,t2) = Data.dest_bal t' 
8760
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    78
      val terms1 = Data.dest_sum t1
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    79
      and terms2 = Data.dest_sum t2
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    80
      val u = find_common (terms1,terms2)
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    81
      val (n1, terms1') = Data.find_first_coeff u terms1
9139453d7033 now works for coefficients, not just for numerals
paulson
parents: 8736
diff changeset
    82
      and (n2, terms2') = Data.find_first_coeff u terms2
14387
e96d5c42c4b0 Polymorphic treatment of binary arithmetic using axclasses
paulson
parents: 13484
diff changeset
    83
      and T = Term.fastype_of u
e96d5c42c4b0 Polymorphic treatment of binary arithmetic using axclasses
paulson
parents: 13484
diff changeset
    84
      fun newshape (i,terms) = Data.mk_sum T (Data.mk_coeff(i,u)::terms)
8779
2d4afbc46801 various bug fixes
paulson
parents: 8772
diff changeset
    85
      val reshape =  (*Move i*u to the front and put j*u into standard form
2d4afbc46801 various bug fixes
paulson
parents: 8772
diff changeset
    86
		       i + #m + j + k == #m + i + (j + k) *)
8772
ebb07113c4f7 inserted triviality check
paulson
parents: 8760
diff changeset
    87
	    if n1=0 orelse n2=0 then   (*trivial, so do nothing*)
ebb07113c4f7 inserted triviality check
paulson
parents: 8760
diff changeset
    88
		raise TERM("cancel_numerals", []) 
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    89
	    else Data.prove_conv [Data.norm_tac ss] thy hyps xs
9191
300bd596d696 now freezes Vars in order to prevent errors in cases like these:
paulson
parents: 8799
diff changeset
    90
			(t', 
8772
ebb07113c4f7 inserted triviality check
paulson
parents: 8760
diff changeset
    91
			 Data.mk_bal (newshape(n1,terms1'), 
8779
2d4afbc46801 various bug fixes
paulson
parents: 8772
diff changeset
    92
				      newshape(n2,terms2')))
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
    93
  in
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    94
      Option.map (Data.simplify_meta_eq ss)
8799
89e9deef4bcb simprocs now simplify the RHS of their result
paulson
parents: 8779
diff changeset
    95
       (if n2<=n1 then 
89e9deef4bcb simprocs now simplify the RHS of their result
paulson
parents: 8779
diff changeset
    96
	    Data.prove_conv 
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    97
	       [Data.trans_tac ss reshape, rtac Data.bal_add1 1,
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
    98
		Data.numeral_simp_tac ss] thy hyps xs
9191
300bd596d696 now freezes Vars in order to prevent errors in cases like these:
paulson
parents: 8799
diff changeset
    99
	       (t', Data.mk_bal (newshape(n1-n2,terms1'), 
14387
e96d5c42c4b0 Polymorphic treatment of binary arithmetic using axclasses
paulson
parents: 13484
diff changeset
   100
				 Data.mk_sum T terms2'))
8799
89e9deef4bcb simprocs now simplify the RHS of their result
paulson
parents: 8779
diff changeset
   101
	else
89e9deef4bcb simprocs now simplify the RHS of their result
paulson
parents: 8779
diff changeset
   102
	    Data.prove_conv 
16973
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
   103
	       [Data.trans_tac ss reshape, rtac Data.bal_add2 1,
b2a894562b8f simprocs: Simplifier.inherit_bounds;
wenzelm
parents: 15965
diff changeset
   104
		Data.numeral_simp_tac ss] thy hyps xs
14387
e96d5c42c4b0 Polymorphic treatment of binary arithmetic using axclasses
paulson
parents: 13484
diff changeset
   105
	       (t', Data.mk_bal (Data.mk_sum T terms1', 
9191
300bd596d696 now freezes Vars in order to prevent errors in cases like these:
paulson
parents: 8799
diff changeset
   106
				 newshape(n2-n1,terms2'))))
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
   107
  end
15531
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 15027
diff changeset
   108
  handle TERM _ => NONE
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 15027
diff changeset
   109
       | TYPE _ => NONE;   (*Typically (if thy doesn't include Numeral)
8779
2d4afbc46801 various bug fixes
paulson
parents: 8772
diff changeset
   110
			     Undeclared type constructor "Numeral.bin"*)
8736
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
   111
0bfd6678a5fa new simprocs for numerals of type "nat"
paulson
parents:
diff changeset
   112
end;