src/HOL/HOL.thy
changeset 66109 e034a563ed7d
parent 63912 9f8325206465
child 66251 cd935b7cb3fb
--- a/src/HOL/HOL.thy	Sat Jun 17 14:52:23 2017 +0200
+++ b/src/HOL/HOL.thy	Sat Jun 17 15:41:19 2017 +0200
@@ -927,6 +927,7 @@
     "\<And>P. (\<exists>x. t = x \<and> P x) = P t"
     "\<And>P. (\<forall>x. x = t \<longrightarrow> P x) = P t"
     "\<And>P. (\<forall>x. t = x \<longrightarrow> P x) = P t"
+    "(\<forall>x. x \<noteq> t) = False"  "(\<forall>x. t \<noteq> x) = False"
   by (blast, blast, blast, blast, blast, iprover+)
 
 lemma disj_absorb: "A \<or> A \<longleftrightarrow> A"