src/HOL/Lattice/Lattice.thy
changeset 12338 de0f4a63baa5
parent 12114 a8e860c86252
child 12818 e7b4c0731d57
equal deleted inserted replaced
12337:7c6a970f0808 12338:de0f4a63baa5
   517       from gh show "g x \<sqsubseteq> h x" ..
   517       from gh show "g x \<sqsubseteq> h x" ..
   518     qed
   518     qed
   519   qed
   519   qed
   520 qed
   520 qed
   521 
   521 
   522 instance fun :: ("term", lattice) lattice
   522 instance fun :: (type, lattice) lattice
   523 proof
   523 proof
   524   fix f g :: "'a \<Rightarrow> 'b::lattice"
   524   fix f g :: "'a \<Rightarrow> 'b::lattice"
   525   show "\<exists>inf. is_inf f g inf" by rule (rule is_inf_fun) (* FIXME @{text "from \<dots> show \<dots> .."} does not work!? unification incompleteness!? *)
   525   show "\<exists>inf. is_inf f g inf" by rule (rule is_inf_fun) (* FIXME @{text "from \<dots> show \<dots> .."} does not work!? unification incompleteness!? *)
   526   show "\<exists>sup. is_sup f g sup" by rule (rule is_sup_fun)
   526   show "\<exists>sup. is_sup f g sup" by rule (rule is_sup_fun)
   527 qed
   527 qed