src/HOL/GCD.thy
changeset 35028 108662d50512
parent 34973 ae634fad947e
child 35216 7641e8d831d2
--- a/src/HOL/GCD.thy	Fri Feb 05 14:33:31 2010 +0100
+++ b/src/HOL/GCD.thy	Fri Feb 05 14:33:50 2010 +0100
@@ -1445,12 +1445,12 @@
 subsubsection {* The complete divisibility lattice *}
 
 
-interpretation gcd_semilattice_nat: lower_semilattice "op dvd" "(%m n::nat. m dvd n & ~ n dvd m)" gcd
+interpretation gcd_semilattice_nat: semilattice_inf "op dvd" "(%m n::nat. m dvd n & ~ n dvd m)" gcd
 proof
   case goal3 thus ?case by(metis gcd_unique_nat)
 qed auto
 
-interpretation lcm_semilattice_nat: upper_semilattice "op dvd" "(%m n::nat. m dvd n & ~ n dvd m)" lcm
+interpretation lcm_semilattice_nat: semilattice_sup "op dvd" "(%m n::nat. m dvd n & ~ n dvd m)" lcm
 proof
   case goal3 thus ?case by(metis lcm_unique_nat)
 qed auto