src/HOL/Real/Float.thy
changeset 20717 2244b0d719a0
parent 20485 3078fd2eec7b
child 20771 89bec28a03c8
--- a/src/HOL/Real/Float.thy	Tue Sep 26 17:33:04 2006 +0200
+++ b/src/HOL/Real/Float.thy	Tue Sep 26 22:37:51 2006 +0200
@@ -3,6 +3,8 @@
     Author: Steven Obua
 *)
 
+header {* Floating Point Representation of the Reals *}
+
 theory Float
 imports Real
 begin