Documentation

Mathlib.Data.PNat.Xgcd

Euclidean algorithm for ℕ #

This file sets up a version of the Euclidean algorithm that only works with natural numbers. Given 0 < a, b, it computes the unique (w, x, y, z, d) such that the following identities hold:

This story is closely related to the structure of SL₂(ℕ) (as a free monoid on two generators) and the theory of continued fractions.

Main declarations #

Notes #

See Nat.Xgcd for a very similar algorithm allowing values in .

structure PNat.XgcdType :

A term of XgcdType is a system of six naturals. They should be thought of as representing the matrix [[w, x], [y, z]] = [[wp + 1, x], [y, zp + 1]] together with the vector [a, b] = [ap + 1, bp + 1].

  • wp : Nat

    wp is a variable which changes through the algorithm.

  • x : Nat

    x satisfies a / d = w + x at the final step.

  • y : Nat

    y satisfies b / d = z + y at the final step.

  • zp : Nat

    zp is a variable which changes through the algorithm.

  • ap : Nat

    ap is a variable which changes through the algorithm.

  • bp : Nat

    bp is a variable which changes through the algorithm.

Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Equations
      Instances For

        The Repr instance converts terms to strings in a way that reflects the matrix/vector interpretation as above.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          def PNat.XgcdType.mk' (w : PNat) (x y : Nat) (z a b : PNat) :

          Another mk using ℕ and ℕ+

          Equations
          Instances For

            w = wp + 1

            Equations
            Instances For

              z = zp + 1

              Equations
              Instances For

                a = ap + 1

                Equations
                Instances For

                  b = bp + 1

                  Equations
                  Instances For

                    r = a % b: remainder

                    Equations
                    Instances For

                      q = ap / bp: quotient

                      Equations
                      Instances For

                        qp = q - 1

                        Equations
                        Instances For

                          The map v gives the product of the matrix [[w, x], [y, z]] = [[wp + 1, x], [y, zp + 1]] and the vector [a, b] = [ap + 1, bp + 1]. The map vp gives [sp, tp] such that v = [sp + 1, tp + 1].

                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For

                            v = [sp + 1, tp + 1], check vp

                            Equations
                            Instances For

                              succ₂ [t.1, t.2] = [t.1.succ, t.2.succ]

                              Equations
                              Instances For

                                IsSpecial holds if the matrix has determinant one.

                                Equations
                                Instances For

                                  IsSpecial' is an alternative of IsSpecial.

                                  Equations
                                  Instances For

                                    IsReduced holds if the two entries in the vector are the same. The reduction algorithm will produce a system with this property, whose product vector is the same as for the original system.

                                    Equations
                                    Instances For

                                      IsReduced' is an alternative of IsReduced.

                                      Equations
                                      Instances For

                                        flip flips the placement of variables during the algorithm.

                                        Equations
                                        • Eq u.flip { wp := u.zp, x := u.y, y := u.x, zp := u.wp, ap := u.bp, bp := u.ap }
                                        Instances For

                                          Properties of division with remainder for a / b.

                                          theorem PNat.XgcdType.qp_eq (u : XgcdType) (hr : Eq u.r 0) :
                                          Eq u.q (HAdd.hAdd u.qp 1)

                                          The following function provides the starting point for our algorithm. We will apply an iterative reduction process to it, which will produce a system satisfying IsReduced. The gcd can be read off from this final system.

                                          Equations
                                          Instances For
                                            theorem PNat.XgcdType.start_v (a b : PNat) :
                                            Eq (start a b).v { fst := a.val, snd := b.val }

                                            finish happens when the reducing process ends.

                                            Equations
                                            Instances For
                                              theorem PNat.XgcdType.finish_v (u : XgcdType) (hr : Eq u.r 0) :
                                              Eq u.finish.v u.v

                                              This is the main reduction step, which is used when u.r ≠ 0, or equivalently b does not divide a.

                                              Equations
                                              Instances For

                                                We will apply the above step recursively. The following result is used to ensure that the process terminates.

                                                theorem PNat.XgcdType.step_v (u : XgcdType) (hr : Ne u.r 0) :
                                                Eq u.step.v u.v.swap

                                                The reduction step does not change the product vector.

                                                @[irreducible]

                                                We can now define the full reduction function, which applies step as long as possible, and then applies finish. Note that the "have" statement puts a fact in the local context, and the equation compiler uses this fact to help construct the full definition in terms of well-founded recursion. The same fact needs to be introduced in all the inductive proofs of properties given below.

                                                Equations
                                                Instances For
                                                  @[irreducible]
                                                  def PNat.xgcd (a b : PNat) :

                                                  Extended Euclidean algorithm

                                                  Equations
                                                  Instances For
                                                    def PNat.gcdD (a b : PNat) :

                                                    gcdD a b = gcd a b

                                                    Equations
                                                    Instances For
                                                      def PNat.gcdW (a b : PNat) :

                                                      Final value of w

                                                      Equations
                                                      Instances For
                                                        def PNat.gcdX (a b : PNat) :

                                                        Final value of x

                                                        Equations
                                                        Instances For
                                                          def PNat.gcdY (a b : PNat) :

                                                          Final value of y

                                                          Equations
                                                          Instances For
                                                            def PNat.gcdZ (a b : PNat) :

                                                            Final value of z

                                                            Equations
                                                            Instances For
                                                              def PNat.gcdA' (a b : PNat) :

                                                              Final value of a / d

                                                              Equations
                                                              Instances For
                                                                def PNat.gcdB' (a b : PNat) :

                                                                Final value of b / d

                                                                Equations
                                                                Instances For
                                                                  theorem PNat.gcdA'_coe (a b : PNat) :
                                                                  Eq (a.gcdA' b).val (HAdd.hAdd (a.gcdW b).val (a.gcdX b))
                                                                  theorem PNat.gcdB'_coe (a b : PNat) :
                                                                  Eq (a.gcdB' b).val (HAdd.hAdd (a.gcdY b) (a.gcdZ b).val)
                                                                  theorem PNat.gcd_props (a b : PNat) :
                                                                  let d := a.gcdD b; let w := a.gcdW b; let x := a.gcdX b; let y := a.gcdY b; let z := a.gcdZ b; let a' := a.gcdA' b; let b' := a.gcdB' b; And (Eq (HMul.hMul w z) (HMul.hMul x y).succPNat) (And (Eq a (HMul.hMul a' d)) (And (Eq b (HMul.hMul b' d)) (And (Eq (HMul.hMul z a') (HMul.hMul x b'.val).succPNat) (And (Eq (HMul.hMul w b') (HMul.hMul y a'.val).succPNat) (And (Eq (HMul.hMul z.val a.val) (HAdd.hAdd (HMul.hMul x b.val) d.val)) (Eq (HMul.hMul w.val b.val) (HAdd.hAdd (HMul.hMul y a.val) d.val)))))))
                                                                  theorem PNat.gcd_eq (a b : PNat) :
                                                                  Eq (a.gcdD b) (a.gcd b)
                                                                  theorem PNat.gcd_det_eq (a b : PNat) :
                                                                  Eq (HMul.hMul (a.gcdW b) (a.gcdZ b)) (HMul.hMul (a.gcdX b) (a.gcdY b)).succPNat
                                                                  theorem PNat.gcd_a_eq (a b : PNat) :
                                                                  Eq a (HMul.hMul (a.gcdA' b) (a.gcd b))
                                                                  theorem PNat.gcd_b_eq (a b : PNat) :
                                                                  Eq b (HMul.hMul (a.gcdB' b) (a.gcd b))
                                                                  theorem PNat.gcd_rel_left' (a b : PNat) :
                                                                  Eq (HMul.hMul (a.gcdZ b) (a.gcdA' b)) (HMul.hMul (a.gcdX b) (a.gcdB' b).val).succPNat
                                                                  theorem PNat.gcd_rel_right' (a b : PNat) :
                                                                  Eq (HMul.hMul (a.gcdW b) (a.gcdB' b)) (HMul.hMul (a.gcdY b) (a.gcdA' b).val).succPNat
                                                                  theorem PNat.gcd_rel_left (a b : PNat) :
                                                                  Eq (HMul.hMul (a.gcdZ b).val a.val) (HAdd.hAdd (HMul.hMul (a.gcdX b) b.val) (a.gcd b).val)
                                                                  theorem PNat.gcd_rel_right (a b : PNat) :
                                                                  Eq (HMul.hMul (a.gcdW b).val b.val) (HAdd.hAdd (HMul.hMul (a.gcdY b) a.val) (a.gcd b).val)