more standard notation (like infix);
authorwenzelm
Sun, 18 Dec 2016 16:13:20 +0100
changeset 64600 86e2f2208a58
parent 64599 80ef54198f44
child 64601 37ce6ceacbb7
more standard notation (like infix);
src/HOL/Nonstandard_Analysis/StarDef.thy
--- a/src/HOL/Nonstandard_Analysis/StarDef.thy	Sun Dec 18 15:53:27 2016 +0100
+++ b/src/HOL/Nonstandard_Analysis/StarDef.thy	Sun Dec 18 16:13:20 2016 +0100
@@ -81,7 +81,7 @@
   by (simp add: FreeUltrafilterNat.proper)
 
 text \<open>Standard principles that play a central role in the transfer tactic.\<close>
-definition Ifun :: "('a \<Rightarrow> 'b) star \<Rightarrow> 'a star \<Rightarrow> 'b star" ("_ \<star> _" [300,301] 300)
+definition Ifun :: "('a \<Rightarrow> 'b) star \<Rightarrow> 'a star \<Rightarrow> 'b star" ("(_ \<star>/ _)" [300, 301] 300)
   where "Ifun f \<equiv>
     \<lambda>x. Abs_star (\<Union>F\<in>Rep_star f. \<Union>X\<in>Rep_star x. starrel``{\<lambda>n. F n (X n)})"