src/HOL/Lattices.thy
changeset 37767 a2b7a20d6ea3
parent 36673 6d25e8dab1e3
child 41075 4bed56dc95fb
equal deleted inserted replaced
37766:a779f463bae4 37767:a2b7a20d6ea3
   621 
   621 
   622 instantiation "fun" :: (type, lattice) lattice
   622 instantiation "fun" :: (type, lattice) lattice
   623 begin
   623 begin
   624 
   624 
   625 definition
   625 definition
   626   inf_fun_eq [code del]: "f \<sqinter> g = (\<lambda>x. f x \<sqinter> g x)"
   626   inf_fun_eq: "f \<sqinter> g = (\<lambda>x. f x \<sqinter> g x)"
   627 
   627 
   628 definition
   628 definition
   629   sup_fun_eq [code del]: "f \<squnion> g = (\<lambda>x. f x \<squnion> g x)"
   629   sup_fun_eq: "f \<squnion> g = (\<lambda>x. f x \<squnion> g x)"
   630 
   630 
   631 instance proof
   631 instance proof
   632 qed (simp_all add: le_fun_def inf_fun_eq sup_fun_eq)
   632 qed (simp_all add: le_fun_def inf_fun_eq sup_fun_eq)
   633 
   633 
   634 end
   634 end