src/HOL/Metis_Examples/Clausify.thy
changeset 42350 128dc0fa87fc
parent 42345 5ecd55993606
child 42747 f132d13fcf75
--- a/src/HOL/Metis_Examples/Clausify.thy	Thu Apr 14 11:24:05 2011 +0200
+++ b/src/HOL/Metis_Examples/Clausify.thy	Thu Apr 14 11:24:05 2011 +0200
@@ -71,6 +71,18 @@
 lemma "r 0 0 \<or> r 1 1 \<or> r 2 2 \<or> r 3 3"
 by (metisFT rax)
 
+lemma "(r 0 0 \<and> r 0 1 \<and> r 0 2 \<and> r 0 3) \<or>
+       (r 1 0 \<and> r 1 1 \<and> r 1 2 \<and> r 1 3) \<or>
+       (r 2 0 \<and> r 2 1 \<and> r 2 2 \<and> r 2 3) \<or>
+       (r 3 0 \<and> r 3 1 \<and> r 3 2 \<and> r 3 3)"
+by (metis rax)
+
+lemma "(r 0 0 \<and> r 0 1 \<and> r 0 2 \<and> r 0 3) \<or>
+       (r 1 0 \<and> r 1 1 \<and> r 1 2 \<and> r 1 3) \<or>
+       (r 2 0 \<and> r 2 1 \<and> r 2 2 \<and> r 2 3) \<or>
+       (r 3 0 \<and> r 3 1 \<and> r 3 2 \<and> r 3 3)"
+by (metisFT rax)
+
 text {* Definitional CNF for goal *}
 
 axiomatization p :: "nat \<Rightarrow> nat \<Rightarrow> bool" where