src/HOL/Lattice/Lattice.thy
changeset 20523 36a59e5d0039
parent 19736 d8d0f8f51d69
child 21210 c17fd2df4e9e
--- a/src/HOL/Lattice/Lattice.thy	Wed Sep 13 00:38:38 2006 +0200
+++ b/src/HOL/Lattice/Lattice.thy	Wed Sep 13 12:05:50 2006 +0200
@@ -519,7 +519,7 @@
   qed
 qed
 
-instance fun :: (type, 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!? *)