author | wenzelm |
Mon, 26 Nov 2012 17:13:44 +0100 | |
changeset 50231 | 81a067b188b8 |
parent 48891 | c0eafbd55de3 |
child 51521 | 36fa825e0ea7 |
child 51539 | 625d2ec0bbff |
permissions | -rw-r--r-- |
28952
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
27964
diff
changeset
|
1 |
theory Real |
29197
6d4cb27ed19c
adapted HOL source structure to distribution layout
haftmann
parents:
29108
diff
changeset
|
2 |
imports RComplete RealVector |
28952
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
27964
diff
changeset
|
3 |
begin |
19640
40ec89317425
added Ferrante and Rackoff Algorithm -- by Amine Chaieb;
wenzelm
parents:
19023
diff
changeset
|
4 |
|
48891 | 5 |
ML_file "Tools/SMT/smt_real.ML" |
6 |
setup SMT_Real.setup |
|
36899
bcd6fce5bf06
layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
boehmes
parents:
35090
diff
changeset
|
7 |
|
19640
40ec89317425
added Ferrante and Rackoff Algorithm -- by Amine Chaieb;
wenzelm
parents:
19023
diff
changeset
|
8 |
end |