CookBook/Recipes/Sat.thy
author Christian Urban <urbanc@in.tum.de>
Thu, 12 Mar 2009 14:25:35 +0000
changeset 171 18f90044c777
parent 127 74846cb0fff9
child 180 9c25418db6f0
permissions -rw-r--r--
simplified antiquotations
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
127
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     1
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     2
theory Sat
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     3
imports Main
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     4
begin
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     5
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     6
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     7
section {* SAT Solver *}
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     8
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     9
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    10
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    11
end
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    12
  
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    13
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    14
74846cb0fff9 updated and added two tentative recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    15