diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Library/Nonpos_Ints.thy --- a/src/HOL/Library/Nonpos_Ints.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Library/Nonpos_Ints.thy Fri Sep 20 19:51:08 2024 +0200 @@ -14,7 +14,7 @@ integers \<^term>\\\) This is useful e.g. for the Gamma function. \ -definition nonpos_Ints ("\\<^sub>\\<^sub>0") where "\\<^sub>\\<^sub>0 = {of_int n |n. n \ 0}" +definition nonpos_Ints (\\\<^sub>\\<^sub>0\) where "\\<^sub>\\<^sub>0 = {of_int n |n. n \ 0}" lemma zero_in_nonpos_Ints [simp,intro]: "0 \ \\<^sub>\\<^sub>0" unfolding nonpos_Ints_def by (auto intro!: exI[of _ "0::int"]) @@ -143,7 +143,7 @@ subsection\Non-negative reals\ -definition nonneg_Reals :: "'a::real_algebra_1 set" ("\\<^sub>\\<^sub>0") +definition nonneg_Reals :: "'a::real_algebra_1 set" (\\\<^sub>\\<^sub>0\) where "\\<^sub>\\<^sub>0 = {of_real r | r. r \ 0}" lemma nonneg_Reals_of_real_iff [simp]: "of_real r \ \\<^sub>\\<^sub>0 \ r \ 0" @@ -210,7 +210,7 @@ subsection\Non-positive reals\ -definition nonpos_Reals :: "'a::real_algebra_1 set" ("\\<^sub>\\<^sub>0") +definition nonpos_Reals :: "'a::real_algebra_1 set" (\\\<^sub>\\<^sub>0\) where "\\<^sub>\\<^sub>0 = {of_real r | r. r \ 0}" lemma nonpos_Reals_of_real_iff [simp]: "of_real r \ \\<^sub>\\<^sub>0 \ r \ 0"