src/HOL/Analysis/Polytope.thy
changeset 69597 ff784d5a5bfb
parent 69508 2a4c8a2a3f8e
child 69661 a03a63b81f44
--- a/src/HOL/Analysis/Polytope.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Analysis/Polytope.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -3072,7 +3072,7 @@
 
 subsection\<open>Simplexes\<close>
 
-text\<open>The notion of n-simplex for integer @{term"n \<ge> -1"}\<close>
+text\<open>The notion of n-simplex for integer \<^term>\<open>n \<ge> -1\<close>\<close>
 definition simplex :: "int \<Rightarrow> 'a::euclidean_space set \<Rightarrow> bool" (infix "simplex" 50)
   where "n simplex S \<equiv> \<exists>C. \<not> affine_dependent C \<and> int(card C) = n + 1 \<and> S = convex hull C"