src/HOL/Real.thy
author wenzelm
Tue, 10 Mar 2009 22:49:56 +0100
changeset 30424 692279df7cc2
parent 29197 6d4cb27ed19c
child 32877 6f09346c7c08
permissions -rw-r--r--
Consts.eq_const is back again (cf. 907da436f8a9) -- required in ProofContext.transfer_syntax to prevent expensive merges of local_consts/global_consts;

theory Real
imports RComplete RealVector
begin

end