src/HOL/Real/HahnBanach/Bounds.thy
changeset 19736 d8d0f8f51d69
parent 16417 9bc16273c2d4
child 21210 c17fd2df4e9e
--- a/src/HOL/Real/HahnBanach/Bounds.thy	Sat May 27 17:42:00 2006 +0200
+++ b/src/HOL/Real/HahnBanach/Bounds.thy	Sat May 27 17:42:02 2006 +0200
@@ -14,12 +14,12 @@
 
 lemmas [elim?] = lub.least lub.upper
 
-constdefs
+definition
   the_lub :: "'a::order set \<Rightarrow> 'a"
-  "the_lub A \<equiv> The (lub A)"
+  "the_lub A = The (lub A)"
 
-syntax (xsymbols)
-  the_lub :: "'a::order set \<Rightarrow> 'a"    ("\<Squnion>_" [90] 90)
+const_syntax (xsymbols)
+  the_lub  ("\<Squnion>_" [90] 90)
 
 lemma the_lub_equality [elim?]:
   includes lub