src/HOL/Decision_Procs/Decision_Procs.thy
author huffman
Mon, 08 Jun 2009 15:46:14 -0700
changeset 31532 43e8d4bfde26
parent 30429 39acdf031548
child 33152 241cfaed158f
permissions -rw-r--r--
generalize lemmas compact_imp_bounded, compact_imp_closed
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
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
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