src/ZF/ex/BinEx.ML
author paulson
Wed, 27 Jan 1999 10:31:31 +0100
changeset 6153 bff90585cce5
parent 5533 bce36a019b03
child 9000 c20d58286a51
permissions -rw-r--r--
new typechecking solver for the simplifier
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     1
(*  Title:      ZF/ex/BinEx.ML
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     2
    ID:         $Id$
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     4
    Copyright   1994  University of Cambridge
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     5
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     6
Examples of performing binary arithmetic by simplification
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     7
*)
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     8
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
     9
context Bin.thy;
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    10
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    11
set proof_timing;
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    12
(*All runtimes below are on a 300MHz Pentium*)
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    13
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    14
Goal "#13  $+  #19 = #32";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    15
by (Simp_tac 1);    (*0 secs*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    16
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    17
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    18
Goal "#1234  $+  #5678 = #6912";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    19
by (Simp_tac 1);    (*190 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    20
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    21
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    22
Goal "#1359  $+  #-2468 = #-1109";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    23
by (Simp_tac 1);    (*160 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    24
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    25
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    26
Goal "#93746  $+  #-46375 = #47371";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    27
by (Simp_tac 1);    (*300 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    28
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    29
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    30
Goal "$~ #65745 = #-65745";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    31
by (Simp_tac 1);    (*80 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    32
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    33
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    34
(* negation of ~54321 *)
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    35
Goal "$~ #-54321 = #54321";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    36
by (Simp_tac 1);    (*90 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    37
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    38
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    39
Goal "#13  $*  #19 = #247";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    40
by (Simp_tac 1);    (*110 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    41
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    42
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    43
Goal "#-84  $*  #51 = #-4284";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    44
by (Simp_tac 1);    (*210 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    45
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    46
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    47
(*The worst case for 8-bit operands *)
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    48
Goal "#255  $*  #255 = #65025";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    49
by (Simp_tac 1);    (*730 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    50
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    51
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    52
Goal "#1359  $*  #-2468 = #-3354012";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    53
by (Simp_tac 1);    (*1.04 secs*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    54
result();