| author | paulson | 
| Tue, 01 May 2001 17:16:32 +0200 | |
| changeset 11276 | f8353c722d4e | 
| parent 9410 | 612ee826a409 | 
| child 11488 | 4ff900551340 | 
| permissions | -rw-r--r-- | 
| 6905 | 1 | (* Title: HOL/Numeral.thy | 
| 2 | ID: $Id$ | |
| 3 | Author: Larry Paulson and Markus Wenzel | |
| 4 | ||
| 9410 
612ee826a409
removed selector syntax -- improper tuples are broken beyond repair :-(
 wenzelm parents: 
9358diff
changeset | 5 | Generic numerals represented as twos-complement bit strings. | 
| 6905 | 6 | *) | 
| 7 | ||
| 8 | theory Numeral = Datatype | |
| 9035 | 9 | files "Tools/numeral_syntax.ML": | 
| 6905 | 10 | |
| 11 | datatype | |
| 12 | bin = Pls | |
| 13 | | Min | |
| 9358 
973672495414
added syntax for proper / improper selector functions;
 wenzelm parents: 
9035diff
changeset | 14 | | Bit bin bool (infixl "BIT" 90) | 
| 6905 | 15 | |
| 16 | axclass | |
| 9035 | 17 | number < "term" (*for numeric types: nat, int, real, ...*) | 
| 6905 | 18 | |
| 19 | consts | |
| 9035 | 20 | number_of :: "bin => 'a::number" | 
| 6905 | 21 | |
| 22 | syntax | |
| 9358 
973672495414
added syntax for proper / improper selector functions;
 wenzelm parents: 
9035diff
changeset | 23 |   "_Numeral" :: "xnum => 'a"    ("_")
 | 
| 6905 | 24 | |
| 9035 | 25 | setup NumeralSyntax.setup | 
| 6905 | 26 | |
| 9035 | 27 | end |