src/HOL/Real/Real.thy
author huffman
Sat, 16 Sep 2006 19:12:03 +0200
changeset 20554 c433e78d4203
parent 20505 1e223f64bd59
child 23454 c54975167be9
permissions -rw-r--r--
define new constant of_real for class real_algebra_1; define set Reals as range of_real; add lemmas about of_real and Reals


(* $Id$ *)

theory Real
imports ContNotDenum Ferrante_Rackoff RealVector
begin
end