Documentation

Mathlib.Tactic.ModCases

mod_cases tactic #

The mod_cases tactic does case disjunction on e % n, where e : ℤ or e : ℕ, to yield n new subgoals corresponding to the possible values of e modulo n.

def Mathlib.Tactic.ModCases.IntMod.OnModCases (n : ) (a : ) (lb : ) (p : Sort u_1) :
Sort (imax 1 u_1)

OnModCases n a lb p represents a partial proof by cases that there exists 0 ≤ z < n such that a ≡ z (mod n). It asserts that if ∃ z, lb ≤ z < n ∧ a ≡ z (mod n) holds, then p (where p is the current goal).

Equations
Instances For
    @[inline]

    The first theorem we apply says that ∃ z, 0 ≤ z < n ∧ a ≡ z (mod n). The actual mathematical content of the proof is here.

    Equations
    Instances For
      @[inline]

      The end point is that once we have reduced to ∃ z, n ≤ z < n ∧ a ≡ z (mod n) there are no more cases to consider.

      Equations
      Instances For
        @[inline]

        The successor case decomposes ∃ z, b ≤ z < n ∧ a ≡ z (mod n) into a ≡ b (mod n) ∨ ∃ z, b+1 ≤ z < n ∧ a ≡ z (mod n), and the a ≡ b (mod n) → p case becomes a subgoal.

        Equations
        Instances For
          partial def Mathlib.Tactic.ModCases.IntMod.proveOnModCases {u : Lean.Level} (n : Q()) (a : Q()) (b : Q()) (p : Q(Sort u)) :

          Proves an expression of the form OnModCases n a b p where n and b are raw nat literals and b ≤ n. Returns the list of subgoals ?gi : a ≡ i [ZMOD n] → p.

          Int case of mod_cases h : e % n.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def Mathlib.Tactic.ModCases.NatMod.OnModCases (n : ) (a : ) (lb : ) (p : Sort u_1) :
            Sort (imax 1 u_1)

            OnModCases n a lb p represents a partial proof by cases that there exists 0 ≤ m < n such that a ≡ m (mod n). It asserts that if ∃ m, lb ≤ m < n ∧ a ≡ m (mod n) holds, then p (where p is the current goal).

            Equations
            Instances For
              @[inline]

              The first theorem we apply says that ∃ m, 0 ≤ m < n ∧ a ≡ m (mod n). The actual mathematical content of the proof is here.

              Equations
              Instances For
                @[inline]

                The end point is that once we have reduced to ∃ m, n ≤ m < n ∧ a ≡ m (mod n) there are no more cases to consider.

                Equations
                Instances For
                  @[inline]

                  The successor case decomposes ∃ m, b ≤ m < n ∧ a ≡ m (mod n) into a ≡ b (mod n) ∨ ∃ m, b+1 ≤ m < n ∧ a ≡ m (mod n), and the a ≡ b (mod n) → p case becomes a subgoal.

                  Equations
                  Instances For
                    partial def Mathlib.Tactic.ModCases.NatMod.proveOnModCases {u : Lean.Level} (n : Q()) (a : Q()) (b : Q()) (p : Q(Sort u)) :

                    Proves an expression of the form OnModCases n a b p where n and b are raw nat literals and b ≤ n. Returns the list of subgoals ?gi : a ≡ i [MOD n] → p.

                    Nat case of mod_cases h : e % n.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      • The tactic mod_cases h : e % 3 will perform a case disjunction on e. If e : ℤ, then it will yield subgoals containing the assumptions h : e ≡ 0 [ZMOD 3], h : e ≡ 1 [ZMOD 3], h : e ≡ 2 [ZMOD 3] respectively. If e : ℕ instead, then it works similarly, except with [MOD 3] instead of [ZMOD 3].
                      • In general, mod_cases h : e % n works when n is a positive numeral and e is an expression of type or .
                      • If h is omitted as in mod_cases e % n, it will be default-named H.
                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For