src/HOL/Decision_Procs/Decision_Procs.thy
author wenzelm
Mon, 16 Mar 2009 18:24:30 +0100
changeset 30549 d2d7874648bd
parent 30429 39acdf031548
child 33152 241cfaed158f
permissions -rw-r--r--
simplified method setup;

header {* Various decision procedures. typically involving reflection *}

theory Decision_Procs
imports Cooper Ferrack MIR Approximation Dense_Linear_Order "ex/Approximation_Ex" "ex/Dense_Linear_Order_Ex"
begin

end