src/HOL/Proofs/Extraction/QuotRem.thy
changeset 67320 6afba546f0e5
parent 66453 cc19f7ca2ed6
equal deleted inserted replaced
67319:07176d5b81d5 67320:6afba546f0e5
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Quotient and remainder\<close>
     5 section \<open>Quotient and remainder\<close>
     6 
     6 
     7 theory QuotRem
     7 theory QuotRem
     8 imports "HOL-Library.Old_Datatype" Util
     8 imports Util "HOL-Library.Realizers"
     9 begin
     9 begin
    10 
    10 
    11 text \<open>Derivation of quotient and remainder using program extraction.\<close>
    11 text \<open>Derivation of quotient and remainder using program extraction.\<close>
    12 
    12 
    13 theorem division: "\<exists>r q. a = Suc b * q + r \<and> r \<le> b"
    13 theorem division: "\<exists>r q. a = Suc b * q + r \<and> r \<le> b"