src/HOL/Lattice/Lattice.thy
changeset 12338 de0f4a63baa5
parent 12114 a8e860c86252
child 12818 e7b4c0731d57
--- a/src/HOL/Lattice/Lattice.thy	Sat Dec 01 18:51:46 2001 +0100
+++ b/src/HOL/Lattice/Lattice.thy	Sat Dec 01 18:52:32 2001 +0100
@@ -519,7 +519,7 @@
   qed
 qed
 
-instance fun :: ("term", lattice) lattice
+instance fun :: (type, lattice) lattice
 proof
   fix f g :: "'a \<Rightarrow> 'b::lattice"
   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!? *)