| author | paulson |
| Tue, 06 May 2003 10:40:43 +0200 | |
| changeset 13963 | ba7aa8c426ad |
| parent 13958 | c1c67582c9b5 |
| child 14425 | 0a76d4633bb6 |
| permissions | -rw-r--r-- |
(* Title: IntFloor.thy Author: Jacques D. Fleuriot Copyright: 2001,2002 University of Edinburgh Description: Floor and ceiling operations over reals *) IntFloor = Integration + constdefs floor :: real => int "floor r == (LEAST n. r < real (n + (1::int)))" ceiling :: real => int "ceiling r == - floor (- r)" end