src/HOL/Decision_Procs/Decision_Procs.thy
author bulwahn
Tue, 27 Oct 2009 09:03:56 +0100
changeset 33254 d0c00b81db1d
parent 33152 241cfaed158f
child 33356 9157d0f9f00e
permissions -rw-r--r--
hiding randompred definitions
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
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
384e47590e7f added Decision_Procs.thy
haftmann
parents:
diff changeset
     3
theory Decision_Procs
33152
241cfaed158f Add a quantifier elimination for parametric linear arithmetic over ordered fields (parameters are multivariate polynomials)
chaieb
parents: 30429
diff changeset
     4
imports Cooper Ferrack MIR Approximation Dense_Linear_Order "ex/Approximation_Ex" "ex/Dense_Linear_Order_Ex" Parametric_Ferrante_Rackoff
29825
384e47590e7f added Decision_Procs.thy
haftmann
parents:
diff changeset
     5
begin
384e47590e7f added Decision_Procs.thy
haftmann
parents:
diff changeset
     6
384e47590e7f added Decision_Procs.thy
haftmann
parents:
diff changeset
     7
end