src/HOL/Hyperreal/IntFloor.thy
author paulson
Mon, 05 May 2003 18:23:40 +0200
changeset 13958 c1c67582c9b5
child 14425 0a76d4633bb6
permissions -rw-r--r--
New material on integration, etc. Moving Hyperreal/ex to directory Complex

(*  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