doc-src/TutorialI/Types/Overloading2.thy
author nipkow
Mon, 23 Oct 2000 20:58:12 +0200
changeset 10305 adff80268127
child 10328 bf33cbd76c05
permissions -rw-r--r--
*** empty log message ***

(*<*)theory Overloading2 = Overloading1:(*>*)

text{*
Of course this is not the only possible definition of the two relations.
Componentwise
*}

instance list :: (ordrel)ordrel
by intro_classes

defs (overloaded)
le_list_def: "xs <<= (ys::'a::ordrel list) \<equiv>
              size xs = size ys \<and> (\<forall>i<size xs. xs!i <<= ys!i)"

text{*
%However, we retract the componetwise comparison of lists and return

Note: only one definition because based on name.
*}
(*<*)end(*>*)