HomeHome Intuitionistic Logic Explorer
Theorem List (p. 142 of 145)
< Previous  Next >
Bad symbols? Try the
GIF version.

Mirrors  >  Metamath Home Page  >  ILE Home Page  >  Theorem List Contents  >  Recent Proofs       This page: Page List

Theorem List for Intuitionistic Logic Explorer - 14101-14200   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremlgsdir2 14101 The Legendre symbol is completely multiplicative at 2. (Contributed by Mario Carneiro, 4-Feb-2015.)
((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ) → ((𝐴 · 𝐵) /L 2) = ((𝐴 /L 2) · (𝐵 /L 2)))
 
Theoremlgsdirprm 14102 The Legendre symbol is completely multiplicative at the primes. See theorem 9.3 in [ApostolNT] p. 180. (Contributed by Mario Carneiro, 4-Feb-2015.) (Proof shortened by AV, 18-Mar-2022.)
((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ 𝑃 ∈ ℙ) → ((𝐴 · 𝐵) /L 𝑃) = ((𝐴 /L 𝑃) · (𝐵 /L 𝑃)))
 
Theoremlgsdir 14103 The Legendre symbol is completely multiplicative in its left argument. Generalization of theorem 9.9(a) in [ApostolNT] p. 188 (which assumes that 𝐴 and 𝐵 are odd positive integers). (Contributed by Mario Carneiro, 4-Feb-2015.)
(((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ (𝐴 ≠ 0 ∧ 𝐵 ≠ 0)) → ((𝐴 · 𝐵) /L 𝑁) = ((𝐴 /L 𝑁) · (𝐵 /L 𝑁)))
 
Theoremlgsdilem2 14104* Lemma for lgsdi 14105. (Contributed by Mario Carneiro, 4-Feb-2015.)
(𝜑𝐴 ∈ ℤ)    &   (𝜑𝑀 ∈ ℤ)    &   (𝜑𝑁 ∈ ℤ)    &   (𝜑𝑀 ≠ 0)    &   (𝜑𝑁 ≠ 0)    &   𝐹 = (𝑛 ∈ ℕ ↦ if(𝑛 ∈ ℙ, ((𝐴 /L 𝑛)↑(𝑛 pCnt 𝑀)), 1))       (𝜑 → (seq1( · , 𝐹)‘(abs‘𝑀)) = (seq1( · , 𝐹)‘(abs‘(𝑀 · 𝑁))))
 
Theoremlgsdi 14105 The Legendre symbol is completely multiplicative in its right argument. Generalization of theorem 9.9(b) in [ApostolNT] p. 188 (which assumes that 𝑀 and 𝑁 are odd positive integers). (Contributed by Mario Carneiro, 5-Feb-2015.)
(((𝐴 ∈ ℤ ∧ 𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ (𝑀 ≠ 0 ∧ 𝑁 ≠ 0)) → (𝐴 /L (𝑀 · 𝑁)) = ((𝐴 /L 𝑀) · (𝐴 /L 𝑁)))
 
Theoremlgsne0 14106 The Legendre symbol is nonzero (and hence equal to 1 or -1) precisely when the arguments are coprime. (Contributed by Mario Carneiro, 5-Feb-2015.)
((𝐴 ∈ ℤ ∧ 𝑁 ∈ ℤ) → ((𝐴 /L 𝑁) ≠ 0 ↔ (𝐴 gcd 𝑁) = 1))
 
Theoremlgsabs1 14107 The Legendre symbol is nonzero (and hence equal to 1 or -1) precisely when the arguments are coprime. (Contributed by Mario Carneiro, 5-Feb-2015.)
((𝐴 ∈ ℤ ∧ 𝑁 ∈ ℤ) → ((abs‘(𝐴 /L 𝑁)) = 1 ↔ (𝐴 gcd 𝑁) = 1))
 
Theoremlgssq 14108 The Legendre symbol at a square is equal to 1. Together with lgsmod 14094 this implies that the Legendre symbol takes value 1 at every quadratic residue. (Contributed by Mario Carneiro, 5-Feb-2015.) (Revised by AV, 20-Jul-2021.)
(((𝐴 ∈ ℤ ∧ 𝐴 ≠ 0) ∧ 𝑁 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((𝐴↑2) /L 𝑁) = 1)
 
Theoremlgssq2 14109 The Legendre symbol at a square is equal to 1. (Contributed by Mario Carneiro, 5-Feb-2015.)
((𝐴 ∈ ℤ ∧ 𝑁 ∈ ℕ ∧ (𝐴 gcd 𝑁) = 1) → (𝐴 /L (𝑁↑2)) = 1)
 
Theoremlgsprme0 14110 The Legendre symbol at any prime (even at 2) is 0 iff the prime does not divide the first argument. See definition in [ApostolNT] p. 179. (Contributed by AV, 20-Jul-2021.)
((𝐴 ∈ ℤ ∧ 𝑃 ∈ ℙ) → ((𝐴 /L 𝑃) = 0 ↔ (𝐴 mod 𝑃) = 0))
 
Theorem1lgs 14111 The Legendre symbol at 1. See example 1 in [ApostolNT] p. 180. (Contributed by Mario Carneiro, 28-Apr-2016.)
(𝑁 ∈ ℤ → (1 /L 𝑁) = 1)
 
Theoremlgs1 14112 The Legendre symbol at 1. See definition in [ApostolNT] p. 188. (Contributed by Mario Carneiro, 28-Apr-2016.)
(𝐴 ∈ ℤ → (𝐴 /L 1) = 1)
 
Theoremlgsmodeq 14113 The Legendre (Jacobi) symbol is preserved under reduction mod 𝑛 when 𝑛 is odd. Theorem 9.9(c) in [ApostolNT] p. 188. (Contributed by AV, 20-Jul-2021.)
((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ (𝑁 ∈ ℕ ∧ ¬ 2 ∥ 𝑁)) → ((𝐴 mod 𝑁) = (𝐵 mod 𝑁) → (𝐴 /L 𝑁) = (𝐵 /L 𝑁)))
 
Theoremlgsmulsqcoprm 14114 The Legendre (Jacobi) symbol is preserved under multiplication with a square of an integer coprime to the second argument. Theorem 9.9(d) in [ApostolNT] p. 188. (Contributed by AV, 20-Jul-2021.)
(((𝐴 ∈ ℤ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℤ ∧ 𝐵 ≠ 0) ∧ (𝑁 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1)) → (((𝐴↑2) · 𝐵) /L 𝑁) = (𝐵 /L 𝑁))
 
Theoremlgsdirnn0 14115 Variation on lgsdir 14103 valid for all 𝐴, 𝐵 but only for positive 𝑁. (The exact location of the failure of this law is for 𝐴 = 0, 𝐵 < 0, 𝑁 = -1 in which case (0 /L -1) = 1 but (𝐵 /L -1) = -1.) (Contributed by Mario Carneiro, 28-Apr-2016.)
((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ 𝑁 ∈ ℕ0) → ((𝐴 · 𝐵) /L 𝑁) = ((𝐴 /L 𝑁) · (𝐵 /L 𝑁)))
 
Theoremlgsdinn0 14116 Variation on lgsdi 14105 valid for all 𝑀, 𝑁 but only for positive 𝐴. (The exact location of the failure of this law is for 𝐴 = -1, 𝑀 = 0, and some 𝑁 in which case (-1 /L 0) = 1 but (-1 /L 𝑁) = -1 when -1 is not a quadratic residue mod 𝑁.) (Contributed by Mario Carneiro, 28-Apr-2016.)
((𝐴 ∈ ℕ0𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝐴 /L (𝑀 · 𝑁)) = ((𝐴 /L 𝑀) · (𝐴 /L 𝑁)))
 
10.2.2  All primes 4n+1 are the sum of two squares
 
Theorem2sqlem1 14117* Lemma for 2sq . (Contributed by Mario Carneiro, 19-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))       (𝐴𝑆 ↔ ∃𝑥 ∈ ℤ[i] 𝐴 = ((abs‘𝑥)↑2))
 
Theorem2sqlem2 14118* Lemma for 2sq . (Contributed by Mario Carneiro, 19-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))       (𝐴𝑆 ↔ ∃𝑥 ∈ ℤ ∃𝑦 ∈ ℤ 𝐴 = ((𝑥↑2) + (𝑦↑2)))
 
Theoremmul2sq 14119 Fibonacci's identity (actually due to Diophantus). The product of two sums of two squares is also a sum of two squares. We can take advantage of Gaussian integers here to trivialize the proof. (Contributed by Mario Carneiro, 19-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))       ((𝐴𝑆𝐵𝑆) → (𝐴 · 𝐵) ∈ 𝑆)
 
Theorem2sqlem3 14120 Lemma for 2sqlem5 14122. (Contributed by Mario Carneiro, 20-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   (𝜑𝑁 ∈ ℕ)    &   (𝜑𝑃 ∈ ℙ)    &   (𝜑𝐴 ∈ ℤ)    &   (𝜑𝐵 ∈ ℤ)    &   (𝜑𝐶 ∈ ℤ)    &   (𝜑𝐷 ∈ ℤ)    &   (𝜑 → (𝑁 · 𝑃) = ((𝐴↑2) + (𝐵↑2)))    &   (𝜑𝑃 = ((𝐶↑2) + (𝐷↑2)))    &   (𝜑𝑃 ∥ ((𝐶 · 𝐵) + (𝐴 · 𝐷)))       (𝜑𝑁𝑆)
 
Theorem2sqlem4 14121 Lemma for 2sqlem5 14122. (Contributed by Mario Carneiro, 20-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   (𝜑𝑁 ∈ ℕ)    &   (𝜑𝑃 ∈ ℙ)    &   (𝜑𝐴 ∈ ℤ)    &   (𝜑𝐵 ∈ ℤ)    &   (𝜑𝐶 ∈ ℤ)    &   (𝜑𝐷 ∈ ℤ)    &   (𝜑 → (𝑁 · 𝑃) = ((𝐴↑2) + (𝐵↑2)))    &   (𝜑𝑃 = ((𝐶↑2) + (𝐷↑2)))       (𝜑𝑁𝑆)
 
Theorem2sqlem5 14122 Lemma for 2sq . If a number that is a sum of two squares is divisible by a prime that is a sum of two squares, then the quotient is a sum of two squares. (Contributed by Mario Carneiro, 20-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   (𝜑𝑁 ∈ ℕ)    &   (𝜑𝑃 ∈ ℙ)    &   (𝜑 → (𝑁 · 𝑃) ∈ 𝑆)    &   (𝜑𝑃𝑆)       (𝜑𝑁𝑆)
 
Theorem2sqlem6 14123* Lemma for 2sq . If a number that is a sum of two squares is divisible by a number whose prime divisors are all sums of two squares, then the quotient is a sum of two squares. (Contributed by Mario Carneiro, 20-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   (𝜑𝐴 ∈ ℕ)    &   (𝜑𝐵 ∈ ℕ)    &   (𝜑 → ∀𝑝 ∈ ℙ (𝑝𝐵𝑝𝑆))    &   (𝜑 → (𝐴 · 𝐵) ∈ 𝑆)       (𝜑𝐴𝑆)
 
Theorem2sqlem7 14124* Lemma for 2sq . (Contributed by Mario Carneiro, 19-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   𝑌 = {𝑧 ∣ ∃𝑥 ∈ ℤ ∃𝑦 ∈ ℤ ((𝑥 gcd 𝑦) = 1 ∧ 𝑧 = ((𝑥↑2) + (𝑦↑2)))}       𝑌 ⊆ (𝑆 ∩ ℕ)
 
Theorem2sqlem8a 14125* Lemma for 2sqlem8 14126. (Contributed by Mario Carneiro, 4-Jun-2016.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   𝑌 = {𝑧 ∣ ∃𝑥 ∈ ℤ ∃𝑦 ∈ ℤ ((𝑥 gcd 𝑦) = 1 ∧ 𝑧 = ((𝑥↑2) + (𝑦↑2)))}    &   (𝜑 → ∀𝑏 ∈ (1...(𝑀 − 1))∀𝑎𝑌 (𝑏𝑎𝑏𝑆))    &   (𝜑𝑀𝑁)    &   (𝜑𝑁 ∈ ℕ)    &   (𝜑𝑀 ∈ (ℤ‘2))    &   (𝜑𝐴 ∈ ℤ)    &   (𝜑𝐵 ∈ ℤ)    &   (𝜑 → (𝐴 gcd 𝐵) = 1)    &   (𝜑𝑁 = ((𝐴↑2) + (𝐵↑2)))    &   𝐶 = (((𝐴 + (𝑀 / 2)) mod 𝑀) − (𝑀 / 2))    &   𝐷 = (((𝐵 + (𝑀 / 2)) mod 𝑀) − (𝑀 / 2))       (𝜑 → (𝐶 gcd 𝐷) ∈ ℕ)
 
Theorem2sqlem8 14126* Lemma for 2sq . (Contributed by Mario Carneiro, 20-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   𝑌 = {𝑧 ∣ ∃𝑥 ∈ ℤ ∃𝑦 ∈ ℤ ((𝑥 gcd 𝑦) = 1 ∧ 𝑧 = ((𝑥↑2) + (𝑦↑2)))}    &   (𝜑 → ∀𝑏 ∈ (1...(𝑀 − 1))∀𝑎𝑌 (𝑏𝑎𝑏𝑆))    &   (𝜑𝑀𝑁)    &   (𝜑𝑁 ∈ ℕ)    &   (𝜑𝑀 ∈ (ℤ‘2))    &   (𝜑𝐴 ∈ ℤ)    &   (𝜑𝐵 ∈ ℤ)    &   (𝜑 → (𝐴 gcd 𝐵) = 1)    &   (𝜑𝑁 = ((𝐴↑2) + (𝐵↑2)))    &   𝐶 = (((𝐴 + (𝑀 / 2)) mod 𝑀) − (𝑀 / 2))    &   𝐷 = (((𝐵 + (𝑀 / 2)) mod 𝑀) − (𝑀 / 2))    &   𝐸 = (𝐶 / (𝐶 gcd 𝐷))    &   𝐹 = (𝐷 / (𝐶 gcd 𝐷))       (𝜑𝑀𝑆)
 
Theorem2sqlem9 14127* Lemma for 2sq . (Contributed by Mario Carneiro, 19-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   𝑌 = {𝑧 ∣ ∃𝑥 ∈ ℤ ∃𝑦 ∈ ℤ ((𝑥 gcd 𝑦) = 1 ∧ 𝑧 = ((𝑥↑2) + (𝑦↑2)))}    &   (𝜑 → ∀𝑏 ∈ (1...(𝑀 − 1))∀𝑎𝑌 (𝑏𝑎𝑏𝑆))    &   (𝜑𝑀𝑁)    &   (𝜑𝑀 ∈ ℕ)    &   (𝜑𝑁𝑌)       (𝜑𝑀𝑆)
 
Theorem2sqlem10 14128* Lemma for 2sq . Every factor of a "proper" sum of two squares (where the summands are coprime) is a sum of two squares. (Contributed by Mario Carneiro, 19-Jun-2015.)
𝑆 = ran (𝑤 ∈ ℤ[i] ↦ ((abs‘𝑤)↑2))    &   𝑌 = {𝑧 ∣ ∃𝑥 ∈ ℤ ∃𝑦 ∈ ℤ ((𝑥 gcd 𝑦) = 1 ∧ 𝑧 = ((𝑥↑2) + (𝑦↑2)))}       ((𝐴𝑌𝐵 ∈ ℕ ∧ 𝐵𝐴) → 𝐵𝑆)
 
PART 11  GUIDES AND MISCELLANEA
 
11.1  Guides (conventions, explanations, and examples)
 
11.1.1  Conventions

This section describes the conventions we use. These conventions often refer to existing mathematical practices, which are discussed in more detail in other references. The following sources lay out how mathematics is developed without the law of the excluded middle. Of course, there are a greater number of sources which assume excluded middle and most of what is in them applies here too (especially in a treatment such as ours which is built on first-order logic and set theory, rather than, say, type theory). Studying how a topic is treated in the Metamath Proof Explorer and the references therein is often a good place to start (and is easy to compare with the Intuitionistic Logic Explorer). The textbooks provide a motivation for what we are doing, whereas Metamath lets you see in detail all hidden and implicit steps. Most standard theorems are accompanied by citations. Some closely followed texts include the following:

  • Axioms of propositional calculus - Stanford Encyclopedia of Philosophy or [Heyting].
  • Axioms of predicate calculus - our axioms are adapted from the ones in the Metamath Proof Explorer.
  • Theorems of propositional calculus - [Heyting].
  • Theorems of pure predicate calculus - Metamath Proof Explorer.
  • Theorems of equality and substitution - Metamath Proof Explorer.
  • Axioms of set theory - [Crosilla].
  • Development of set theory - Chapter 10 of [HoTT].
  • Construction of real and complex numbers - Chapter 11 of [HoTT]; [BauerTaylor].
  • Theorems about real numbers - [Geuvers].
 
Theoremconventions 14129 Unless there is a reason to diverge, we follow the conventions of the Metamath Proof Explorer (MPE, set.mm). This list of conventions is intended to be read in conjunction with the corresponding conventions in the Metamath Proof Explorer, and only the differences are described below.
  • Minimizing axioms and the axiom of choice. We prefer proofs that depend on fewer and/or weaker axioms, even if the proofs are longer. In particular, our choice of IZF (Intuitionistic Zermelo-Fraenkel) over CZF (Constructive Zermelo-Fraenkel, a weaker system) was just an expedient choice because IZF is easier to formalize in Metamath. You can find some development using CZF in BJ's mathbox starting at wbd 14220 (and the section header just above it). As for the axiom of choice, the full axiom of choice implies excluded middle as seen at acexmid 5868, although some authors will use countable choice or dependent choice. For example, countable choice or excluded middle is needed to show that the Cauchy reals coincide with the Dedekind reals - Corollary 11.4.3 of [HoTT], p. (varies).
  • Junk/undefined results. Much of the discussion of this topic in the Metamath Proof Explorer applies except that certain techniques are not available to us. For example, the Metamath Proof Explorer will often say "if a function is evaluated within its domain, a certain result follows; if the function is evaluated outside its domain, the same result follows. Since the function must be evaluated within its domain or outside it, the result follows unconditionally" (the use of excluded middle in this argument is perhaps obvious when stated this way). Often, the easiest fix will be to prove we are evaluating functions within their domains, other times it will be possible to use a theorem like relelfvdm 5543 which says that if a function value produces an inhabited set, then the function is being evaluated within its domain.
  • Bibliography references. The bibliography for the Intuitionistic Logic Explorer is separate from the one for the Metamath Proof Explorer but feel free to copy-paste a citation in either direction in order to cite it.

Label naming conventions

Here are a few of the label naming conventions:

  • Suffixes. We follow the conventions of the Metamath Proof Explorer with a few additions. A biconditional in set.mm which is an implication in iset.mm should have a "r" (for the reverse direction), or "i"/"im" (for the forward direction) appended. A theorem in set.mm which has a decidability condition added should add "dc" to the theorem name. A theorem in set.mm where "nonempty class" is changed to "inhabited class" should add "m" (for member) to the theorem name.
  • iset.mm versus set.mm names

    Theorems which are the same as in set.mm should be named the same (that is, where the statement of the theorem is the same; the proof can differ without a new name being called for). Theorems which are different should be named differently (we do have a small number of intentional exceptions to this rule but on the whole it serves us well).

    As for how to choose names so they are different between iset.mm and set.mm, when possible choose a name which reflect the difference in the theorems. For example, if a theorem in set.mm is an equality and the iset.mm analogue is a subset, add "ss" to the iset.mm name. If need be, add "i" to the iset.mm name (usually as a prefix to some portion of the name).

    As with set.mm, we welcome suggestions for better names (such as names which are more consistent with naming conventions).

    We do try to keep set.mm and iset.mm similar where we can. For example, if a theorem exists in both places but the name in set.mm isn't great, we tend to keep that name for iset.mm, or change it in both files together. This is mainly to make it easier to copy theorems, but also to generally help people browse proofs, find theorems, write proofs, etc.

The following table shows some commonly-used abbreviations in labels which are not found in the Metamath Proof Explorer, in alphabetical order. For each abbreviation we provide a mnenomic to help you remember it, the source theorem/assumption defining it, an expression showing what it looks like, whether or not it is a "syntax fragment" (an abbreviation that indicates a particular kind of syntax), and hyperlinks to label examples that use the abbreviation. The abbreviation is bolded if there is a df-NAME definition but the label fragment is not NAME.

For the "g" abbreviation, this is related to the set.mm usage, in which "is a set" conditions are converted from hypotheses to antecedents, but is also used where "is a set" conditions are added relative to similar set.mm theorems.

AbbreviationMnenomic/MeaningSource ExpressionSyntax?Example(s)
apapart df-ap 8529 Yes apadd1 8555, apne 8570
gwith "is a set" condition No 1stvalg 6137, brtposg 6249, setsmsbasg 13646
seq3, sum3recursive sequence df-seqfrec 10432 Yes seq3-1 10446, fsum3 11379
taptight apartness df-tap 7241 Yes df-tap 7241

(Contributed by Jim Kingdon, 24-Feb-2020.) (New usage is discouraged.)

𝜑       𝜑
 
11.1.2  Definitional examples
 
Theoremex-or 14130 Example for ax-io 709. Example by David A. Wheeler. (Contributed by Mario Carneiro, 9-May-2015.)
(2 = 3 ∨ 4 = 4)
 
Theoremex-an 14131 Example for ax-ia1 106. Example by David A. Wheeler. (Contributed by Mario Carneiro, 9-May-2015.)
(2 = 2 ∧ 3 = 3)
 
Theorem1kp2ke3k 14132 Example for df-dec 9374, 1000 + 2000 = 3000.

This proof disproves (by counterexample) the assertion of Hao Wang, who stated, "There is a theorem in the primitive notation of set theory that corresponds to the arithmetic theorem 1000 + 2000 = 3000. The formula would be forbiddingly long... even if (one) knows the definitions and is asked to simplify the long formula according to them, chances are he will make errors and arrive at some incorrect result." (Hao Wang, "Theory and practice in mathematics" , In Thomas Tymoczko, editor, New Directions in the Philosophy of Mathematics, pp 129-152, Birkauser Boston, Inc., Boston, 1986. (QA8.6.N48). The quote itself is on page 140.)

This is noted in Metamath: A Computer Language for Pure Mathematics by Norman Megill (2007) section 1.1.3. Megill then states, "A number of writers have conveyed the impression that the kind of absolute rigor provided by Metamath is an impossible dream, suggesting that a complete, formal verification of a typical theorem would take millions of steps in untold volumes of books... These writers assume, however, that in order to achieve the kind of complete formal verification they desire one must break down a proof into individual primitive steps that make direct reference to the axioms. This is not necessary. There is no reason not to make use of previously proved theorems rather than proving them over and over... A hierarchy of theorems and definitions permits an exponential growth in the formula sizes and primitive proof steps to be described with only a linear growth in the number of symbols used. Of course, this is how ordinary informal mathematics is normally done anyway, but with Metamath it can be done with absolute rigor and precision."

The proof here starts with (2 + 1) = 3, commutes it, and repeatedly multiplies both sides by ten. This is certainly longer than traditional mathematical proofs, e.g., there are a number of steps explicitly shown here to show that we're allowed to do operations such as multiplication. However, while longer, the proof is clearly a manageable size - even though every step is rigorously derived all the way back to the primitive notions of set theory and logic. And while there's a risk of making errors, the many independent verifiers make it much less likely that an incorrect result will be accepted.

This proof heavily relies on the decimal constructor df-dec 9374 developed by Mario Carneiro in 2015. The underlying Metamath language has an intentionally very small set of primitives; it doesn't even have a built-in construct for numbers. Instead, the digits are defined using these primitives, and the decimal constructor is used to make it easy to express larger numbers as combinations of digits.

(Contributed by David A. Wheeler, 29-Jun-2016.) (Shortened by Mario Carneiro using the arithmetic algorithm in mmj2, 30-Jun-2016.)

(1000 + 2000) = 3000
 
Theoremex-fl 14133 Example for df-fl 10256. Example by David A. Wheeler. (Contributed by Mario Carneiro, 18-Jun-2015.)
((⌊‘(3 / 2)) = 1 ∧ (⌊‘-(3 / 2)) = -2)
 
Theoremex-ceil 14134 Example for df-ceil 10257. (Contributed by AV, 4-Sep-2021.)
((⌈‘(3 / 2)) = 2 ∧ (⌈‘-(3 / 2)) = -1)
 
Theoremex-exp 14135 Example for df-exp 10506. (Contributed by AV, 4-Sep-2021.)
((5↑2) = 25 ∧ (-3↑-2) = (1 / 9))
 
Theoremex-fac 14136 Example for df-fac 10690. (Contributed by AV, 4-Sep-2021.)
(!‘5) = 120
 
Theoremex-bc 14137 Example for df-bc 10712. (Contributed by AV, 4-Sep-2021.)
(5C3) = 10
 
Theoremex-dvds 14138 Example for df-dvds 11779: 3 divides into 6. (Contributed by David A. Wheeler, 19-May-2015.)
3 ∥ 6
 
Theoremex-gcd 14139 Example for df-gcd 11927. (Contributed by AV, 5-Sep-2021.)
(-6 gcd 9) = 3
 
PART 12  SUPPLEMENTARY MATERIAL (USERS' MATHBOXES)
 
12.1  Mathboxes for user contributions
 
12.1.1  Mathbox guidelines
 
Theoremmathbox 14140 (This theorem is a dummy placeholder for these guidelines. The label of this theorem, "mathbox", is hard-coded into the Metamath program to identify the start of the mathbox section for web page generation.)

A "mathbox" is a user-contributed section that is maintained by its contributor independently from the main part of iset.mm.

For contributors:

By making a contribution, you agree to release it into the public domain, according to the statement at the beginning of iset.mm.

Guidelines:

Mathboxes in iset.mm follow the same practices as in set.mm, so refer to the mathbox guidelines there for more details.

(Contributed by NM, 20-Feb-2007.) (Revised by the Metamath team, 9-Sep-2023.) (New usage is discouraged.)

𝜑       𝜑
 
12.2  Mathbox for BJ
 
12.2.1  Propositional calculus
 
Theorembj-nnsn 14141 As far as implying a negated formula is concerned, a formula is equivalent to its double negation. (Contributed by BJ, 24-Nov-2023.)
((𝜑 → ¬ 𝜓) ↔ (¬ ¬ 𝜑 → ¬ 𝜓))
 
Theorembj-nnor 14142 Double negation of a disjunction in terms of implication. (Contributed by BJ, 9-Oct-2019.)
(¬ ¬ (𝜑𝜓) ↔ (¬ 𝜑 → ¬ ¬ 𝜓))
 
Theorembj-nnim 14143 The double negation of an implication implies the implication with the consequent doubly negated. (Contributed by BJ, 24-Nov-2023.)
(¬ ¬ (𝜑𝜓) → (𝜑 → ¬ ¬ 𝜓))
 
Theorembj-nnan 14144 The double negation of a conjunction implies the conjunction of the double negations. (Contributed by BJ, 24-Nov-2023.)
(¬ ¬ (𝜑𝜓) → (¬ ¬ 𝜑 ∧ ¬ ¬ 𝜓))
 
Theorembj-nnclavius 14145 Clavius law with doubly negated consequent. (Contributed by BJ, 4-Dec-2023.)
((¬ 𝜑𝜑) → ¬ ¬ 𝜑)
 
Theorembj-imnimnn 14146 If a formula is implied by both a formula and its negation, then it is not refutable. There is another proof using the inference associated with bj-nnclavius 14145 as its last step. (Contributed by BJ, 27-Oct-2024.)
(𝜑𝜓)    &   𝜑𝜓)        ¬ ¬ 𝜓
 
12.2.1.1  Stable formulas

Some of the following theorems, like bj-sttru 14148 or bj-stfal 14150 could be deduced from their analogues for decidability, but stability is not provable from decidability in minimal calculus, so direct proofs have their interest.

 
Theorembj-trst 14147 A provable formula is stable. (Contributed by BJ, 24-Nov-2023.)
(𝜑STAB 𝜑)
 
Theorembj-sttru 14148 The true truth value is stable. (Contributed by BJ, 5-Aug-2024.)
STAB
 
Theorembj-fast 14149 A refutable formula is stable. (Contributed by BJ, 24-Nov-2023.)
𝜑STAB 𝜑)
 
Theorembj-stfal 14150 The false truth value is stable. (Contributed by BJ, 5-Aug-2024.)
STAB
 
Theorembj-nnst 14151 Double negation of stability of a formula. Intuitionistic logic refutes unstability (but does not prove stability) of any formula. This theorem can also be proved in classical refutability calculus (see https://us.metamath.org/mpeuni/bj-peircestab.html) but not in minimal calculus (see https://us.metamath.org/mpeuni/bj-stabpeirce.html). See nnnotnotr 14398 for the version not using the definition of stability. (Contributed by BJ, 9-Oct-2019.) Prove it in ( → , ¬ ) -intuitionistic calculus with definitions (uses of ax-ia1 106, ax-ia2 107, ax-ia3 108 are via sylibr 134, necessary for definition unpackaging), and in ( → , ↔ , ¬ )-intuitionistic calculus, following a discussion with Jim Kingdon. (Revised by BJ, 27-Oct-2024.)
¬ ¬ STAB 𝜑
 
Theorembj-nnbist 14152 If a formula is not refutable, then it is stable if and only if it is provable. By double-negation translation, if 𝜑 is a classical tautology, then ¬ ¬ 𝜑 is an intuitionistic tautology. Therefore, if 𝜑 is a classical tautology, then 𝜑 is intuitionistically equivalent to its stability (and to its decidability, see bj-nnbidc 14165). (Contributed by BJ, 24-Nov-2023.)
(¬ ¬ 𝜑 → (STAB 𝜑𝜑))
 
Theorembj-stst 14153 Stability of a proposition is stable if and only if that proposition is stable. STAB is idempotent. (Contributed by BJ, 9-Oct-2019.)
(STAB STAB 𝜑STAB 𝜑)
 
Theorembj-stim 14154 A conjunction with a stable consequent is stable. See stabnot 833 for negation , bj-stan 14155 for conjunction , and bj-stal 14157 for universal quantification. (Contributed by BJ, 24-Nov-2023.)
(STAB 𝜓STAB (𝜑𝜓))
 
Theorembj-stan 14155 The conjunction of two stable formulas is stable. See bj-stim 14154 for implication, stabnot 833 for negation, and bj-stal 14157 for universal quantification. (Contributed by BJ, 24-Nov-2023.)
((STAB 𝜑STAB 𝜓) → STAB (𝜑𝜓))
 
Theorembj-stand 14156 The conjunction of two stable formulas is stable. Deduction form of bj-stan 14155. Its proof is shorter (when counting all steps, including syntactic steps), so one could prove it first and then bj-stan 14155 from it, the usual way. (Contributed by BJ, 24-Nov-2023.) (Proof modification is discouraged.)
(𝜑STAB 𝜓)    &   (𝜑STAB 𝜒)       (𝜑STAB (𝜓𝜒))
 
Theorembj-stal 14157 The universal quantification of a stable formula is stable. See bj-stim 14154 for implication, stabnot 833 for negation, and bj-stan 14155 for conjunction. (Contributed by BJ, 24-Nov-2023.)
(∀𝑥STAB 𝜑STAB𝑥𝜑)
 
Theorembj-pm2.18st 14158 Clavius law for stable formulas. See pm2.18dc 855. (Contributed by BJ, 4-Dec-2023.)
(STAB 𝜑 → ((¬ 𝜑𝜑) → 𝜑))
 
Theorembj-con1st 14159 Contraposition when the antecedent is a negated stable proposition. See con1dc 856. (Contributed by BJ, 11-Nov-2024.)
(STAB 𝜑 → ((¬ 𝜑𝜓) → (¬ 𝜓𝜑)))
 
12.2.1.2  Decidable formulas
 
Theorembj-trdc 14160 A provable formula is decidable. (Contributed by BJ, 24-Nov-2023.)
(𝜑DECID 𝜑)
 
Theorembj-dctru 14161 The true truth value is decidable. (Contributed by BJ, 5-Aug-2024.)
DECID
 
Theorembj-fadc 14162 A refutable formula is decidable. (Contributed by BJ, 24-Nov-2023.)
𝜑DECID 𝜑)
 
Theorembj-dcfal 14163 The false truth value is decidable. (Contributed by BJ, 5-Aug-2024.)
DECID
 
Theorembj-dcstab 14164 A decidable formula is stable. (Contributed by BJ, 24-Nov-2023.) (Proof modification is discouraged.)
(DECID 𝜑STAB 𝜑)
 
Theorembj-nnbidc 14165 If a formula is not refutable, then it is decidable if and only if it is provable. See also comment of bj-nnbist 14152. (Contributed by BJ, 24-Nov-2023.)
(¬ ¬ 𝜑 → (DECID 𝜑𝜑))
 
Theorembj-nndcALT 14166 Alternate proof of nndc 851. (Proof modification is discouraged.) (New usage is discouraged.) (Contributed by BJ, 9-Oct-2019.)
¬ ¬ DECID 𝜑
 
Theorembj-dcdc 14167 Decidability of a proposition is decidable if and only if that proposition is decidable. DECID is idempotent. (Contributed by BJ, 9-Oct-2019.)
(DECID DECID 𝜑DECID 𝜑)
 
Theorembj-stdc 14168 Decidability of a proposition is stable if and only if that proposition is decidable. In particular, the assumption that every formula is stable implies that every formula is decidable, hence classical logic. (Contributed by BJ, 9-Oct-2019.)
(STAB DECID 𝜑DECID 𝜑)
 
Theorembj-dcst 14169 Stability of a proposition is decidable if and only if that proposition is stable. (Contributed by BJ, 24-Nov-2023.)
(DECID STAB 𝜑STAB 𝜑)
 
12.2.2  Predicate calculus
 
Theorembj-ex 14170* Existential generalization. (Contributed by BJ, 8-Dec-2019.) Proof modification is discouraged because there are shorter proofs, but using less basic results (like exlimiv 1598 and 19.9ht 1641 or 19.23ht 1497). (Proof modification is discouraged.)
(∃𝑥𝜑𝜑)
 
Theorembj-hbalt 14171 Closed form of hbal 1477 (copied from set.mm). (Contributed by BJ, 2-May-2019.)
(∀𝑦(𝜑 → ∀𝑥𝜑) → (∀𝑦𝜑 → ∀𝑥𝑦𝜑))
 
Theorembj-nfalt 14172 Closed form of nfal 1576 (copied from set.mm). (Contributed by BJ, 2-May-2019.) (Proof modification is discouraged.)
(∀𝑥𝑦𝜑 → Ⅎ𝑦𝑥𝜑)
 
Theoremspimd 14173 Deduction form of spim 1738. (Contributed by BJ, 17-Oct-2019.)
(𝜑 → Ⅎ𝑥𝜒)    &   (𝜑 → ∀𝑥(𝑥 = 𝑦 → (𝜓𝜒)))       (𝜑 → (∀𝑥𝜓𝜒))
 
Theorem2spim 14174* Double substitution, as in spim 1738. (Contributed by BJ, 17-Oct-2019.)
𝑥𝜒    &   𝑧𝜒    &   ((𝑥 = 𝑦𝑧 = 𝑡) → (𝜓𝜒))       (∀𝑧𝑥𝜓𝜒)
 
Theoremch2var 14175* Implicit substitution of 𝑦 for 𝑥 and 𝑡 for 𝑧 into a theorem. (Contributed by BJ, 17-Oct-2019.)
𝑥𝜓    &   𝑧𝜓    &   ((𝑥 = 𝑦𝑧 = 𝑡) → (𝜑𝜓))    &   𝜑       𝜓
 
Theoremch2varv 14176* Version of ch2var 14175 with nonfreeness hypotheses replaced with disjoint variable conditions. (Contributed by BJ, 17-Oct-2019.)
((𝑥 = 𝑦𝑧 = 𝑡) → (𝜑𝜓))    &   𝜑       𝜓
 
Theorembj-exlimmp 14177 Lemma for bj-vtoclgf 14184. (Contributed by BJ, 21-Nov-2019.) (Proof modification is discouraged.)
𝑥𝜓    &   (𝜒𝜑)       (∀𝑥(𝜒 → (𝜑𝜓)) → (∃𝑥𝜒𝜓))
 
Theorembj-exlimmpi 14178 Lemma for bj-vtoclgf 14184. (Contributed by BJ, 21-Nov-2019.) (Proof modification is discouraged.)
𝑥𝜓    &   (𝜒𝜑)    &   (𝜒 → (𝜑𝜓))       (∃𝑥𝜒𝜓)
 
Theorembj-sbimedh 14179 A strengthening of sbiedh 1787 (same proof). (Contributed by BJ, 16-Dec-2019.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜒 → ∀𝑥𝜒))    &   (𝜑 → (𝑥 = 𝑦 → (𝜓𝜒)))       (𝜑 → ([𝑦 / 𝑥]𝜓𝜒))
 
Theorembj-sbimeh 14180 A strengthening of sbieh 1790 (same proof). (Contributed by BJ, 16-Dec-2019.)
(𝜓 → ∀𝑥𝜓)    &   (𝑥 = 𝑦 → (𝜑𝜓))       ([𝑦 / 𝑥]𝜑𝜓)
 
Theorembj-sbime 14181 A strengthening of sbie 1791 (same proof). (Contributed by BJ, 16-Dec-2019.)
𝑥𝜓    &   (𝑥 = 𝑦 → (𝜑𝜓))       ([𝑦 / 𝑥]𝜑𝜓)
 
12.2.3  Set theorey miscellaneous
 
Theorembj-el2oss1o 14182 Shorter proof of el2oss1o 6438 using more axioms. (Contributed by BJ, 21-Jan-2024.) (Proof modification is discouraged.) (New usage is discouraged.)
(𝐴 ∈ 2o𝐴 ⊆ 1o)
 
12.2.4  Extensionality

Various utility theorems using FOL and extensionality.

 
Theorembj-vtoclgft 14183 Weakening two hypotheses of vtoclgf 2795. (Contributed by BJ, 21-Nov-2019.)
𝑥𝐴    &   𝑥𝜓    &   (𝑥 = 𝐴𝜑)       (∀𝑥(𝑥 = 𝐴 → (𝜑𝜓)) → (𝐴𝑉𝜓))
 
Theorembj-vtoclgf 14184 Weakening two hypotheses of vtoclgf 2795. (Contributed by BJ, 21-Nov-2019.)
𝑥𝐴    &   𝑥𝜓    &   (𝑥 = 𝐴𝜑)    &   (𝑥 = 𝐴 → (𝜑𝜓))       (𝐴𝑉𝜓)
 
Theoremelabgf0 14185 Lemma for elabgf 2879. (Contributed by BJ, 21-Nov-2019.)
(𝑥 = 𝐴 → (𝐴 ∈ {𝑥𝜑} ↔ 𝜑))
 
Theoremelabgft1 14186 One implication of elabgf 2879, in closed form. (Contributed by BJ, 21-Nov-2019.)
𝑥𝐴    &   𝑥𝜓       (∀𝑥(𝑥 = 𝐴 → (𝜑𝜓)) → (𝐴 ∈ {𝑥𝜑} → 𝜓))
 
Theoremelabgf1 14187 One implication of elabgf 2879. (Contributed by BJ, 21-Nov-2019.)
𝑥𝐴    &   𝑥𝜓    &   (𝑥 = 𝐴 → (𝜑𝜓))       (𝐴 ∈ {𝑥𝜑} → 𝜓)
 
Theoremelabgf2 14188 One implication of elabgf 2879. (Contributed by BJ, 21-Nov-2019.)
𝑥𝐴    &   𝑥𝜓    &   (𝑥 = 𝐴 → (𝜓𝜑))       (𝐴𝐵 → (𝜓𝐴 ∈ {𝑥𝜑}))
 
Theoremelabf1 14189* One implication of elabf 2880. (Contributed by BJ, 21-Nov-2019.)
𝑥𝜓    &   (𝑥 = 𝐴 → (𝜑𝜓))       (𝐴 ∈ {𝑥𝜑} → 𝜓)
 
Theoremelabf2 14190* One implication of elabf 2880. (Contributed by BJ, 21-Nov-2019.)
𝑥𝜓    &   𝐴 ∈ V    &   (𝑥 = 𝐴 → (𝜓𝜑))       (𝜓𝐴 ∈ {𝑥𝜑})
 
Theoremelab1 14191* One implication of elab 2881. (Contributed by BJ, 21-Nov-2019.)
(𝑥 = 𝐴 → (𝜑𝜓))       (𝐴 ∈ {𝑥𝜑} → 𝜓)
 
Theoremelab2a 14192* One implication of elab 2881. (Contributed by BJ, 21-Nov-2019.)
𝐴 ∈ V    &   (𝑥 = 𝐴 → (𝜓𝜑))       (𝜓𝐴 ∈ {𝑥𝜑})
 
Theoremelabg2 14193* One implication of elabg 2883. (Contributed by BJ, 21-Nov-2019.)
(𝑥 = 𝐴 → (𝜓𝜑))       (𝐴𝑉 → (𝜓𝐴 ∈ {𝑥𝜑}))
 
Theorembj-rspgt 14194 Restricted specialization, generalized. Weakens a hypothesis of rspccv 2838 and seems to have a shorter proof. (Contributed by BJ, 21-Nov-2019.)
𝑥𝐴    &   𝑥𝐵    &   𝑥𝜓       (∀𝑥(𝑥 = 𝐴 → (𝜑𝜓)) → (∀𝑥𝐵 𝜑 → (𝐴𝐵𝜓)))
 
Theorembj-rspg 14195 Restricted specialization, generalized. Weakens a hypothesis of rspccv 2838 and seems to have a shorter proof. (Contributed by BJ, 21-Nov-2019.)
𝑥𝐴    &   𝑥𝐵    &   𝑥𝜓    &   (𝑥 = 𝐴 → (𝜑𝜓))       (∀𝑥𝐵 𝜑 → (𝐴𝐵𝜓))
 
Theoremcbvrald 14196* Rule used to change bound variables, using implicit substitution. (Contributed by BJ, 22-Nov-2019.)
𝑥𝜑    &   𝑦𝜑    &   (𝜑 → Ⅎ𝑦𝜓)    &   (𝜑 → Ⅎ𝑥𝜒)    &   (𝜑 → (𝑥 = 𝑦 → (𝜓𝜒)))       (𝜑 → (∀𝑥𝐴 𝜓 ↔ ∀𝑦𝐴 𝜒))
 
Theorembj-intabssel 14197 Version of intss1 3857 using a class abstraction and explicit substitution. (Contributed by BJ, 29-Nov-2019.)
𝑥𝐴       (𝐴𝑉 → ([𝐴 / 𝑥]𝜑 {𝑥𝜑} ⊆ 𝐴))
 
Theorembj-intabssel1 14198 Version of intss1 3857 using a class abstraction and implicit substitution. Closed form of intmin3 3869. (Contributed by BJ, 29-Nov-2019.)
𝑥𝐴    &   𝑥𝜓    &   (𝑥 = 𝐴 → (𝜓𝜑))       (𝐴𝑉 → (𝜓 {𝑥𝜑} ⊆ 𝐴))
 
Theorembj-elssuniab 14199 Version of elssuni 3835 using a class abstraction and explicit substitution. (Contributed by BJ, 29-Nov-2019.)
𝑥𝐴       (𝐴𝑉 → ([𝐴 / 𝑥]𝜑𝐴 {𝑥𝜑}))
 
Theorembj-sseq 14200 If two converse inclusions are characterized each by a formula, then equality is characterized by the conjunction of these formulas. (Contributed by BJ, 30-Nov-2019.)
(𝜑 → (𝜓𝐴𝐵))    &   (𝜑 → (𝜒𝐵𝐴))       (𝜑 → ((𝜓𝜒) ↔ 𝐴 = 𝐵))
    < Previous  Next >

Page List
Jump to page: Contents  1 1-100 2 101-200 3 201-300 4 301-400 5 401-500 6 501-600 7 601-700 8 701-800 9 801-900 10 901-1000 11 1001-1100 12 1101-1200 13 1201-1300 14 1301-1400 15 1401-1500 16 1501-1600 17 1601-1700 18 1701-1800 19 1801-1900 20 1901-2000 21 2001-2100 22 2101-2200 23 2201-2300 24 2301-2400 25 2401-2500 26 2501-2600 27 2601-2700 28 2701-2800 29 2801-2900 30 2901-3000 31 3001-3100 32 3101-3200 33 3201-3300 34 3301-3400 35 3401-3500 36 3501-3600 37 3601-3700 38 3701-3800 39 3801-3900 40 3901-4000 41 4001-4100 42 4101-4200 43 4201-4300 44 4301-4400 45 4401-4500 46 4501-4600 47 4601-4700 48 4701-4800 49 4801-4900 50 4901-5000 51 5001-5100 52 5101-5200 53 5201-5300 54 5301-5400 55 5401-5500 56 5501-5600 57 5601-5700 58 5701-5800 59 5801-5900 60 5901-6000 61 6001-6100 62 6101-6200 63 6201-6300 64 6301-6400 65 6401-6500 66 6501-6600 67 6601-6700 68 6701-6800 69 6801-6900 70 6901-7000 71 7001-7100 72 7101-7200 73 7201-7300 74 7301-7400 75 7401-7500 76 7501-7600 77 7601-7700 78 7701-7800 79 7801-7900 80 7901-8000 81 8001-8100 82 8101-8200 83 8201-8300 84 8301-8400 85 8401-8500 86 8501-8600 87 8601-8700 88 8701-8800 89 8801-8900 90 8901-9000 91 9001-9100 92 9101-9200 93 9201-9300 94 9301-9400 95 9401-9500 96 9501-9600 97 9601-9700 98 9701-9800 99 9801-9900 100 9901-10000 101 10001-10100 102 10101-10200 103 10201-10300 104 10301-10400 105 10401-10500 106 10501-10600 107 10601-10700 108 10701-10800 109 10801-10900 110 10901-11000 111 11001-11100 112 11101-11200 113 11201-11300 114 11301-11400 115 11401-11500 116 11501-11600 117 11601-11700 118 11701-11800 119 11801-11900 120 11901-12000 121 12001-12100 122 12101-12200 123 12201-12300 124 12301-12400 125 12401-12500 126 12501-12600 127 12601-12700 128 12701-12800 129 12801-12900 130 12901-13000 131 13001-13100 132 13101-13200 133 13201-13300 134 13301-13400 135 13401-13500 136 13501-13600 137 13601-13700 138 13701-13800 139 13801-13900 140 13901-14000 141 14001-14100 142 14101-14200 143 14201-14300 144 14301-14400 145 14401-14485
  Copyright terms: Public domain < Previous  Next >