src/HOL/Real/Real.thy
author urbanc
Tue, 13 Dec 2005 18:11:21 +0100
changeset 18396 b3e7da94b51f
parent 15536 3ce1cb7a24f0
child 19023 5652a536b7e8
permissions -rw-r--r--
added a fresh_left lemma that contains all instantiation for the various atom-types.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
15536
3ce1cb7a24f0 starting to get rid of sumr
nipkow
parents: 14374
diff changeset
     1
theory Real
3ce1cb7a24f0 starting to get rid of sumr
nipkow
parents: 14374
diff changeset
     2
imports RComplete RealPow
3ce1cb7a24f0 starting to get rid of sumr
nipkow
parents: 14374
diff changeset
     3
begin
3ce1cb7a24f0 starting to get rid of sumr
nipkow
parents: 14374
diff changeset
     4
end