--- a/src/HOL/Algebra/Exact_Sequence.thy Wed Oct 09 22:01:33 2024 +0200
+++ b/src/HOL/Algebra/Exact_Sequence.thy Wed Oct 09 23:38:29 2024 +0200
@@ -22,7 +22,7 @@
abbreviation exact_seq_arrow ::
"('a \<Rightarrow> 'a) \<Rightarrow> 'a monoid list \<times> ('a \<Rightarrow> 'a) list \<Rightarrow> 'a monoid \<Rightarrow> 'a monoid list \<times> ('a \<Rightarrow> 'a) list"
- (\<open>(3_ / \<longlongrightarrow>\<index> _)\<close> [1000, 60])
+ (\<open>(\<open>indent=3 notation=\<open>mixfix exact_seq\<close>\<close>_ / \<longlongrightarrow>\<index> _)\<close> [1000, 60])
where "exact_seq_arrow f t G \<equiv> (G # (fst t), f # (snd t))"