src/HOL/ex/SAT_Examples.thy
changeset 67613 ce654b0e6d69
parent 61933 cf58b5b794b2
child 69597 ff784d5a5bfb
--- a/src/HOL/ex/SAT_Examples.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/ex/SAT_Examples.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -76,7 +76,7 @@
 
 text \<open>eta-Equivalence\<close>
 
-lemma "(ALL x. P x) | ~ All P"
+lemma "(\<forall>x. P x) \<or> \<not> All P"
 by sat
 
 declare [[sat_trace = false]]