aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Euclid_def.v
blob: 292816f4542c4ca2a713770f0c8601a5477d6c17 (plain)
1
2
3
4
5
6
7

(* $Id$ *)

Require Export Mult.

Inductive diveucl [a,b:nat] : Set 
      := divex : (q,r:nat)(gt b r)->(a=(plus (mult q b) r))->(diveucl a b).