doc-src/TutorialI/Advanced/Partial.thy
changeset 17914 99ead7a7eb42
parent 15904 a6fb4ddc05c7
child 19248 25bb0a883ac5
equal deleted inserted replaced
17913:4159e1523ad8 17914:99ead7a7eb42
     1 (*<*)theory Partial = While_Combinator:(*>*)
     1 (*<*)theory Partial imports While_Combinator begin(*>*)
     2 
     2 
     3 text{*\noindent Throughout this tutorial, we have emphasized
     3 text{*\noindent Throughout this tutorial, we have emphasized
     4 that all functions in HOL are total.  We cannot hope to define
     4 that all functions in HOL are total.  We cannot hope to define
     5 truly partial functions, but must make them total.  A straightforward
     5 truly partial functions, but must make them total.  A straightforward
     6 method is to lift the result type of the function from $\tau$ to
     6 method is to lift the result type of the function from $\tau$ to