clauses for iff-introduction, unfortunately useless
authorpaulson
Wed, 01 Nov 2006 15:51:11 +0100
changeset 21137 8a1d62375ff8
parent 21136 85fd05aaf737
child 21138 afdd72fc6c4f
clauses for iff-introduction, unfortunately useless
src/HOL/Reconstruction.thy
--- a/src/HOL/Reconstruction.thy	Wed Nov 01 15:50:19 2006 +0100
+++ b/src/HOL/Reconstruction.thy	Wed Nov 01 15:51:11 2006 +0100
@@ -71,6 +71,16 @@
 apply (simp add: COMBB_def) 
 done
 
+text{*These two represent the equivalence between Boolean equality and iff.
+They can't be converted to clauses automatically, as the iff would be 
+expanded...*}
+
+lemma iff_positive: "P | Q | P=Q"
+by blast
+
+lemma iff_negative: "~P | ~Q | P=Q"
+by blast
+
 use "Tools/res_axioms.ML"
 use "Tools/res_hol_clause.ML"
 use "Tools/res_atp.ML"