| Thu, 18 Apr 2013 17:07:01 +0200 | 
wenzelm | 
simplifier uses proper Proof.context instead of historic type simpset;
 | 
file |
diff |
annotate
 | 
| Fri, 27 Jul 2012 17:57:31 +0200 | 
huffman | 
give Nat_Arith simprocs proper name bindings by using simproc_setup
 | 
file |
diff |
annotate
 | 
| Fri, 27 Jul 2012 15:42:39 +0200 | 
huffman | 
replace abel_cancel simprocs with functionally equivalent, but simpler and faster ones
 | 
file |
diff |
annotate
 | 
| Fri, 20 Jul 2012 10:53:25 +0200 | 
huffman | 
make nat_cancel_sums simprocs robust in the presence of schematic variables; add regression tests
 | 
file |
diff |
annotate
 | 
| Sun, 25 Mar 2012 20:15:39 +0200 | 
huffman | 
merged fork with new numeral representation (see NEWS)
 | 
file |
diff |
annotate
 | 
| Tue, 17 Jan 2012 16:30:54 +0100 | 
huffman | 
factor-cancellation simprocs now call the full simplifier to prove that factors are non-zero
 | 
file |
diff |
annotate
 | 
| Wed, 16 Nov 2011 15:20:27 +0100 | 
huffman | 
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 | 
file |
diff |
annotate
 | 
| Fri, 11 Nov 2011 12:30:28 +0100 | 
huffman | 
abel_cancel.ML: avoid canceling zeros, which would cause the simproc to return a trivial rewrite;
 | 
file |
diff |
annotate
 | 
| Fri, 11 Nov 2011 11:30:31 +0100 | 
huffman | 
use simproc_setup for the remaining nat_numeral simprocs
 | 
file |
diff |
annotate
 | 
| Fri, 11 Nov 2011 11:11:03 +0100 | 
huffman | 
use simproc_setup for more nat_numeral simprocs; add simproc tests
 | 
file |
diff |
annotate
 | 
| Wed, 09 Nov 2011 15:33:24 +0100 | 
huffman | 
tune post-processing of simproc-generated rules so they won't produce Numeral0 or Numeral1
 | 
file |
diff |
annotate
 | 
| Wed, 09 Nov 2011 11:44:42 +0100 | 
huffman | 
use simproc_setup for some nat_numeral simprocs; add simproc tests
 | 
file |
diff |
annotate
 | 
| Wed, 09 Nov 2011 10:58:08 +0100 | 
huffman | 
add ring_char_0 class constraints to several simprocs (internal proofs of #n ~= 0 fail for type
 | 
file |
diff |
annotate
 | 
| Fri, 28 Oct 2011 10:33:23 +0200 | 
huffman | 
ex/Simproc_Tests.thy: remove duplicate simprocs
 | 
file |
diff |
annotate
 | 
| Fri, 28 Oct 2011 11:02:27 +0200 | 
huffman | 
use simproc_setup for cancellation simprocs, to get proper name bindings
 | 
file |
diff |
annotate
 | 
| Thu, 27 Oct 2011 07:46:57 +0200 | 
huffman | 
fix bug in cancel_factor simprocs so they will work on goals like 'x * y < x * z' where the common term is already on the left
 | 
file |
diff |
annotate
 | 
| Fri, 21 Oct 2011 08:42:11 +0200 | 
huffman | 
add HOL/ex/Simproc_Tests.thy: testing for Tools/numeral_simprocs.ML
 | 
file |
diff |
annotate
 |