src/HOL/Decision_Procs/Decision_Procs.thy
author bulwahn
Mon, 11 May 2009 09:18:42 +0200
changeset 31106 9a1178204dc0
parent 30429 39acdf031548
child 33152 241cfaed158f
permissions -rw-r--r--
Added pred_code command

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