src/HOL/Multivariate_Analysis/Brouwer_Fixpoint.thy
changeset 62843 313d3b697c9a
parent 62393 a620a8756b7c
child 62948 7700f467892b
--- a/src/HOL/Multivariate_Analysis/Brouwer_Fixpoint.thy	Mon Apr 04 09:45:04 2016 +0200
+++ b/src/HOL/Multivariate_Analysis/Brouwer_Fixpoint.thy	Mon Apr 04 16:52:56 2016 +0100
@@ -1781,7 +1781,7 @@
 
 definition "retraction s t r \<longleftrightarrow> t \<subseteq> s \<and> continuous_on s r \<and> r ` s \<subseteq> t \<and> (\<forall>x\<in>t. r x = x)"
 
-definition retract_of (infixl "retract'_of" 12)
+definition retract_of (infixl "retract'_of" 50)
   where "(t retract_of s) \<longleftrightarrow> (\<exists>r. retraction s t r)"
 
 lemma retraction_idempotent: "retraction s t r \<Longrightarrow> x \<in> s \<Longrightarrow>  r (r x) = r x"