src/HOL/Real/Real.thy
author wenzelm
Mon, 17 Oct 2005 23:10:15 +0200
changeset 17877 67d5ab1cb0d8
parent 15536 3ce1cb7a24f0
child 19023 5652a536b7e8
permissions -rw-r--r--
Simplifier.inherit_context instead of Simplifier.inherit_bounds;
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