(* Title: HOLCF/fun2.thy ID: $Id$ Author: Franz Regensburger Copyright 1993 Technische Universitaet MuenchenClass Instance =>::(term,po)poDefiniton of least element*)Fun2 = Fun1 + (* default class is still term !*)(* Witness for the above arity axiom is fun1.ML *)arities fun :: (term,po)poconsts UU_fun :: "'a::term => 'b::pcpo"rules(* instance of << for type ['a::term => 'b::po] *)inst_fun_po "(op <<)::['a=>'b::po,'a=>'b::po ]=>bool = less_fun"(* definitions *)(* The least element in type 'a::term => 'b::pcpo *)UU_fun_def "UU_fun == (% x.UU)"end