doc-src/TutorialI/Types/Overloading1.thy
changeset 10885 90695f46440b
parent 10396 5ab08609e6c8
child 11161 166f7d87b37f
equal deleted inserted replaced
10884:2995639c6a09 10885:90695f46440b
     1 (*<*)theory Overloading1 = Main:(*>*)
     1 (*<*)theory Overloading1 = Main:(*>*)
     2 
     2 
     3 subsubsection{*Controlled overloading with type classes*}
     3 subsubsection{*Controlled Overloading with Type Classes*}
     4 
     4 
     5 text{*
     5 text{*
     6 We now start with the theory of ordering relations, which we want to phrase
     6 We now start with the theory of ordering relations, which we want to phrase
     7 in terms of the two binary symbols @{text"<<"} and @{text"<<="}: they have
     7 in terms of the two binary symbols @{text"<<"} and @{text"<<="}: they have
     8 been chosen to avoid clashes with @{text"<"} and @{text"\<le>"} in theory @{text
     8 been chosen to avoid clashes with @{text"<"} and @{text"\<le>"} in theory @{text