src/HOL/Lattice/CompleteLattice.thy
changeset 21404 eb85850d3eb7
parent 21210 c17fd2df4e9e
child 23373 ead82c82da9e
--- a/src/HOL/Lattice/CompleteLattice.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/Lattice/CompleteLattice.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -32,13 +32,14 @@
 *}
 
 definition
-  Meet :: "'a::complete_lattice set \<Rightarrow> 'a"
+  Meet :: "'a::complete_lattice set \<Rightarrow> 'a" where
   "Meet A = (THE inf. is_Inf A inf)"
-  Join :: "'a::complete_lattice set \<Rightarrow> 'a"
+definition
+  Join :: "'a::complete_lattice set \<Rightarrow> 'a" where
   "Join A = (THE sup. is_Sup A sup)"
 
 notation (xsymbols)
-  Meet  ("\<Sqinter>_" [90] 90)
+  Meet  ("\<Sqinter>_" [90] 90) and
   Join  ("\<Squnion>_" [90] 90)
 
 text {*
@@ -143,9 +144,10 @@
 *}
 
 definition
-  bottom :: "'a::complete_lattice"    ("\<bottom>")
+  bottom :: "'a::complete_lattice"    ("\<bottom>") where
   "\<bottom> = \<Sqinter>UNIV"
-  top :: "'a::complete_lattice"    ("\<top>")
+definition
+  top :: "'a::complete_lattice"    ("\<top>") where
   "\<top> = \<Squnion>UNIV"
 
 lemma bottom_least [intro?]: "\<bottom> \<sqsubseteq> x"