src/HOL/Induct/SList.thy
changeset 81128 5b201b24d99b
parent 80914 d97fdabd9e2b
child 81133 072cc2a92ba3
--- a/src/HOL/Induct/SList.thy	Tue Oct 08 15:02:17 2024 +0200
+++ b/src/HOL/Induct/SList.thy	Tue Oct 08 15:44:11 2024 +0200
@@ -83,9 +83,7 @@
 no_translations
   "[x, xs]" == "x#[xs]"
   "[x]" == "x#[]"
-no_notation
-  Nil  (\<open>[]\<close>) and
-  Cons (infixr \<open>#\<close> 65)
+no_notation Nil  (\<open>[]\<close>) and Cons  (infixr \<open>#\<close> 65)
 
 definition
   Nil       :: "'a list"                               (\<open>[]\<close>) where