| author | nipkow |
| Fri, 13 Mar 2009 12:32:29 +0100 | |
| changeset 30502 | b80d2621caee |
| parent 30429 | 39acdf031548 |
| child 33152 | 241cfaed158f |
| permissions | -rw-r--r-- |
|
30429
39acdf031548
moved Decision_Procs examples to Decision_Procs/ex
haftmann
parents:
29825
diff
changeset
|
1 |
header {* Various decision procedures. typically involving reflection *}
|
|
39acdf031548
moved Decision_Procs examples to Decision_Procs/ex
haftmann
parents:
29825
diff
changeset
|
2 |
|
| 29825 | 3 |
theory Decision_Procs |
|
30429
39acdf031548
moved Decision_Procs examples to Decision_Procs/ex
haftmann
parents:
29825
diff
changeset
|
4 |
imports Cooper Ferrack MIR Approximation Dense_Linear_Order "ex/Approximation_Ex" "ex/Dense_Linear_Order_Ex" |
| 29825 | 5 |
begin |
6 |
||
7 |
end |