src/HOL/GCD.thy
changeset 61169 4de9ff3ea29a
parent 60758 d8d85a8172b5
child 61566 c3d6e570ccef
equal deleted inserted replaced
61168:dcdfb6355a05 61169:4de9ff3ea29a
  1973   complete_lattice Gcd Lcm gcd Rings.dvd "\<lambda>m n. m dvd n \<and> \<not> n dvd m" lcm 1 "0::nat"
  1973   complete_lattice Gcd Lcm gcd Rings.dvd "\<lambda>m n. m dvd n \<and> \<not> n dvd m" lcm 1 "0::nat"
  1974 where "Inf.INFIMUM Gcd A f = Gcd (f ` A :: nat set)"
  1974 where "Inf.INFIMUM Gcd A f = Gcd (f ` A :: nat set)"
  1975   and "Sup.SUPREMUM Lcm A f = Lcm (f ` A)"
  1975   and "Sup.SUPREMUM Lcm A f = Lcm (f ` A)"
  1976 proof -
  1976 proof -
  1977   show "class.complete_lattice Gcd Lcm gcd Rings.dvd (\<lambda>m n. m dvd n \<and> \<not> n dvd m) lcm 1 (0::nat)"
  1977   show "class.complete_lattice Gcd Lcm gcd Rings.dvd (\<lambda>m n. m dvd n \<and> \<not> n dvd m) lcm 1 (0::nat)"
  1978     by default (auto simp add: Gcd_nat_def Lcm_nat_empty Lcm_nat_infinite)
  1978     by standard (auto simp add: Gcd_nat_def Lcm_nat_empty Lcm_nat_infinite)
  1979   then interpret gcd_lcm_complete_lattice_nat:
  1979   then interpret gcd_lcm_complete_lattice_nat:
  1980     complete_lattice Gcd Lcm gcd Rings.dvd "\<lambda>m n. m dvd n \<and> \<not> n dvd m" lcm 1 "0::nat" .
  1980     complete_lattice Gcd Lcm gcd Rings.dvd "\<lambda>m n. m dvd n \<and> \<not> n dvd m" lcm 1 "0::nat" .
  1981   from gcd_lcm_complete_lattice_nat.INF_def show "Inf.INFIMUM Gcd A f = Gcd (f ` A)" .
  1981   from gcd_lcm_complete_lattice_nat.INF_def show "Inf.INFIMUM Gcd A f = Gcd (f ` A)" .
  1982   from gcd_lcm_complete_lattice_nat.SUP_def show "Sup.SUPREMUM Lcm A f = Lcm (f ` A)" .
  1982   from gcd_lcm_complete_lattice_nat.SUP_def show "Sup.SUPREMUM Lcm A f = Lcm (f ` A)" .
  1983 qed
  1983 qed