src/HOL/Number_Theory/Cong.thy
changeset 71546 4dd5dadfc87d
parent 69597 ff784d5a5bfb
child 76224 64e8d4afcf10
--- a/src/HOL/Number_Theory/Cong.thy	Fri Mar 13 16:04:27 2020 +0100
+++ b/src/HOL/Number_Theory/Cong.thy	Fri Mar 13 16:12:50 2020 +0100
@@ -37,10 +37,10 @@
 context unique_euclidean_semiring
 begin
 
-definition cong :: "'a \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"  (\<open>(1[_ = _] '(()mod _'))\<close>)
+definition cong :: "'a \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"  (\<open>(1[_ = _] '(' mod _'))\<close>)
   where "cong b c a \<longleftrightarrow> b mod a = c mod a"
   
-abbreviation notcong :: "'a \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"  (\<open>(1[_ \<noteq> _] '(()mod _'))\<close>)
+abbreviation notcong :: "'a \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"  (\<open>(1[_ \<noteq> _] '(' mod _'))\<close>)
   where "notcong b c a \<equiv> \<not> cong b c a"
 
 lemma cong_refl [simp]: