src/HOL/Analysis/Euclidean_Space.thy
changeset 81142 6ad2c917dd2e
parent 80914 d97fdabd9e2b
child 82522 62afd98e3f3e
--- a/src/HOL/Analysis/Euclidean_Space.thy	Wed Oct 09 22:01:33 2024 +0200
+++ b/src/HOL/Analysis/Euclidean_Space.thy	Wed Oct 09 23:38:29 2024 +0200
@@ -33,7 +33,7 @@
   assumes euclidean_all_zero_iff:
     "(\<forall>u\<in>Basis. inner x u = 0) \<longleftrightarrow> (x = 0)"
 
-syntax "_type_dimension" :: "type \<Rightarrow> nat"  (\<open>(1DIM/(1'(_')))\<close>)
+syntax "_type_dimension" :: "type \<Rightarrow> nat"  (\<open>(\<open>indent=1 notation=\<open>mixfix type dimension\<close>\<close>DIM/(1'(_')))\<close>)
 syntax_consts "_type_dimension" \<rightleftharpoons> card
 translations "DIM('a)" \<rightharpoonup> "CONST card (CONST Basis :: 'a set)"
 typed_print_translation \<open>