src/ZF/ex/BinEx.ML
author wenzelm
Thu, 06 Jul 2000 18:12:17 +0200
changeset 9274 21c302a2fd9a
parent 9000 c20d58286a51
child 9548 15bee2731e43
permissions -rw-r--r--
tuned msgs;
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
(*All runtimes below are on a 300MHz Pentium*)
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    12
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    13
Goal "#13  $+  #19 = #32";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    14
by (Simp_tac 1);    (*0 secs*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    15
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    16
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    17
Goal "#1234  $+  #5678 = #6912";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    18
by (Simp_tac 1);    (*190 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    19
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    20
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    21
Goal "#1359  $+  #-2468 = #-1109";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    22
by (Simp_tac 1);    (*160 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    23
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    24
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    25
Goal "#93746  $+  #-46375 = #47371";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    26
by (Simp_tac 1);    (*300 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    27
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    28
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    29
Goal "$~ #65745 = #-65745";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    30
by (Simp_tac 1);    (*80 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    31
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    32
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    33
(* negation of ~54321 *)
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    34
Goal "$~ #-54321 = #54321";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    35
by (Simp_tac 1);    (*90 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    36
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    37
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    38
Goal "#13  $*  #19 = #247";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    39
by (Simp_tac 1);    (*110 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    40
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    41
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    42
Goal "#-84  $*  #51 = #-4284";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    43
by (Simp_tac 1);    (*210 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    44
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    45
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    46
(*The worst case for 8-bit operands *)
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    47
Goal "#255  $*  #255 = #65025";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    48
by (Simp_tac 1);    (*730 msec*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    49
result();
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    50
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    51
Goal "#1359  $*  #-2468 = #-3354012";
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 5533
diff changeset
    52
by (Simp_tac 1);    (*1.04 secs*)
5533
bce36a019b03 re-organized for the new directory Integ
paulson
parents:
diff changeset
    53
result();