src/HOL/Library/Perm.thy
changeset 67399 eab6ce8368fa
parent 64911 f0e07600de47
child 68406 6beb45f6cf67
--- a/src/HOL/Library/Perm.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Library/Perm.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -27,7 +27,7 @@
 setup_lifting type_definition_perm
 
 notation "apply" (infixl "\<langle>$\<rangle>" 999)
-no_notation "apply" ("op \<langle>$\<rangle>")
+no_notation "apply" ("(\<langle>$\<rangle>)")
 
 lemma bij_apply [simp]:
   "bij (apply f)"
@@ -804,7 +804,7 @@
   notation swap       ("\<langle>_\<leftrightarrow>_\<rangle>")
   notation cycle      ("\<langle>_\<rangle>")
   notation "apply"    (infixl "\<langle>$\<rangle>" 999)
-  no_notation "apply" ("op \<langle>$\<rangle>")
+  no_notation "apply" ("(\<langle>$\<rangle>)")
 end
 
 unbundle no_permutation_syntax