equal
deleted
inserted
replaced
1 (* Title: ZF/ex/BinEx.ML |
1 (* Title: ZF/ex/BinEx.thy |
2 ID: $Id$ |
|
3 Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
2 Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
4 Copyright 1994 University of Cambridge |
3 Copyright 1994 University of Cambridge |
5 |
4 |
6 Examples of performing binary arithmetic by simplification |
5 Examples of performing binary arithmetic by simplification. |
7 *) |
6 *) |
8 |
7 |
9 theory BinEx imports Main begin |
8 theory BinEx imports Main begin |
10 (*All runtimes below are on a 300MHz Pentium*) |
9 (*All runtimes below are on a 300MHz Pentium*) |
11 |
10 |