src/HOL/Library/Z2.thy
changeset 73535 0f33c7031ec9
parent 72082 41393ecb57ac
child 73682 78044b2f001c
--- a/src/HOL/Library/Z2.thy	Mon Apr 05 22:46:41 2021 +0200
+++ b/src/HOL/Library/Z2.thy	Tue Apr 06 18:12:20 2021 +0000
@@ -224,7 +224,7 @@
   where [simp]: \<open>NOT b = of_bool (even b)\<close> for b :: bit
 
 instance
-  by standard simp_all
+  by standard auto
 
 end