| author | wenzelm | 
| Mon, 25 Jun 2012 11:07:51 +0200 | |
| changeset 48120 | 9fe0e71052a0 | 
| parent 36899 | bcd6fce5bf06 | 
| child 48891 | c0eafbd55de3 | 
| permissions | -rw-r--r-- | 
| 28952 
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
 haftmann parents: 
27964diff
changeset | 1 | theory Real | 
| 29197 
6d4cb27ed19c
adapted HOL source structure to distribution layout
 haftmann parents: 
29108diff
changeset | 2 | imports RComplete RealVector | 
| 36899 
bcd6fce5bf06
layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
 boehmes parents: 
35090diff
changeset | 3 | uses "Tools/SMT/smt_real.ML" | 
| 28952 
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
 haftmann parents: 
27964diff
changeset | 4 | begin | 
| 19640 
40ec89317425
added Ferrante and Rackoff Algorithm -- by Amine Chaieb;
 wenzelm parents: 
19023diff
changeset | 5 | |
| 36899 
bcd6fce5bf06
layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
 boehmes parents: 
35090diff
changeset | 6 | setup {* SMT_Real.setup *}
 | 
| 
bcd6fce5bf06
layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
 boehmes parents: 
35090diff
changeset | 7 | |
| 19640 
40ec89317425
added Ferrante and Rackoff Algorithm -- by Amine Chaieb;
 wenzelm parents: 
19023diff
changeset | 8 | end |