src/HOL/Real/Real.thy
author wenzelm
Wed, 13 Apr 2005 18:49:42 +0200
changeset 15723 5b594d6ec919
parent 15536 3ce1cb7a24f0
child 19023 5652a536b7e8
permissions -rw-r--r--
*** MESSAGE REFERS TO PREVIOUS VERSION *** added declared_tyname/const and read_tyname/const; removed certify_tyname/const; added prep_ext_merge, nontriv_merge kept internal; efficient subsig test;
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