src/HOL/ex/SAT_Examples.thy
changeset 61933 cf58b5b794b2
parent 61343 5b5656a63bd6
child 67613 ce654b0e6d69
equal deleted inserted replaced
61932:2e48182cc82c 61933:cf58b5b794b2
   275 shows "False"
   275 shows "False"
   276 using assms
   276 using assms
   277 (*
   277 (*
   278 by sat
   278 by sat
   279 *)
   279 *)
   280 by rawsat  -- \<open>this is without CNF conversion\<close>
   280 by rawsat  \<comment> \<open>this is without CNF conversion\<close>
   281 
   281 
   282 (* Translated from TPTP problem library: MSC007-1.008.dimacs *)
   282 (* Translated from TPTP problem library: MSC007-1.008.dimacs *)
   283 
   283 
   284 lemma assumes 1: "x0 | x1 | x2 | x3 | x4 | x5 | x6"
   284 lemma assumes 1: "x0 | x1 | x2 | x3 | x4 | x5 | x6"
   285 and 2: "x7 | x8 | x9 | x10 | x11 | x12 | x13"
   285 and 2: "x7 | x8 | x9 | x10 | x11 | x12 | x13"
   488 shows "False"
   488 shows "False"
   489 using assms
   489 using assms
   490 (*
   490 (*
   491 by sat
   491 by sat
   492 *)
   492 *)
   493 by rawsat  -- \<open>this is without CNF conversion\<close>
   493 by rawsat  \<comment> \<open>this is without CNF conversion\<close>
   494 
   494 
   495 (* Old sequent clause representation ("[c_i, p, ~q, \<dots>] \<turnstile> False"):
   495 (* Old sequent clause representation ("[c_i, p, ~q, \<dots>] \<turnstile> False"):
   496    sat, zchaff_with_proofs: 8705 resolution steps in
   496    sat, zchaff_with_proofs: 8705 resolution steps in
   497                             +++ User 1.154  All 1.189 secs
   497                             +++ User 1.154  All 1.189 secs
   498    sat, minisat_with_proofs: 40790 resolution steps in
   498    sat, minisat_with_proofs: 40790 resolution steps in