src/HOL/ex/Bit_Lists.thy
changeset 70340 7383930fc946
parent 70339 e939ea997f5f
child 70353 7aa64296b9b0
--- a/src/HOL/ex/Bit_Lists.thy	Fri Jun 14 08:34:27 2019 +0000
+++ b/src/HOL/ex/Bit_Lists.thy	Fri Jun 14 08:34:27 2019 +0000
@@ -25,7 +25,7 @@
 
 end
 
-class semiring_bits = semiring_parity +
+class semiring_bits = unique_euclidean_semiring_with_nat +
   assumes half_measure: "a div 2 \<noteq> a \<Longrightarrow> euclidean_size (a div 2) < euclidean_size a"
   \<comment> \<open>It is not clear whether this could be derived from already existing assumptions.\<close>
 begin
@@ -82,7 +82,7 @@
   "of_unsigned (bits_of n) = n" for n :: nat
   using of_unsigned_bits_of_nat [of n, where ?'a = nat] by simp
 
-class ring_bits = ring_parity + semiring_bits
+class ring_bits = unique_euclidean_ring_with_nat + semiring_bits
 begin
 
 lemma bits_of_minus_1 [simp]: