src/HOL/Lattices_Big.thy
changeset 67036 783c901a62cb
parent 66425 8756322dc5de
child 67169 1fabca1c2199
--- a/src/HOL/Lattices_Big.thy	Tue Nov 07 14:52:27 2017 +0100
+++ b/src/HOL/Lattices_Big.thy	Wed Nov 08 21:01:53 2017 +0100
@@ -837,7 +837,7 @@
 
 syntax
   "_arg_min" :: "('a \<Rightarrow> 'b) \<Rightarrow> pttrn \<Rightarrow> bool \<Rightarrow> 'a"
-    ("(3ARG'_MIN _ _./ _)" [0, 0, 10] 10)
+    ("(3ARG'_MIN _ _./ _)" [1000, 0, 10] 10)
 translations
   "ARG_MIN f x. P" \<rightleftharpoons> "CONST arg_min f (\<lambda>x. P)"
 
@@ -945,7 +945,7 @@
 
 syntax
   "_arg_max" :: "('a \<Rightarrow> 'b) \<Rightarrow> pttrn \<Rightarrow> bool \<Rightarrow> 'a"
-    ("(3ARG'_MAX _ _./ _)" [0, 0, 10] 10)
+    ("(3ARG'_MAX _ _./ _)" [1000, 0, 10] 10)
 translations
   "ARG_MAX f x. P" \<rightleftharpoons> "CONST arg_max f (\<lambda>x. P)"