MPE Home Metamath Proof Explorer < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  MPE Home  >  Th. List  >  odzval Structured version   Visualization version   GIF version

Theorem odzval 16420
Description: Value of the order function. This is a function of functions; the inner argument selects the base (i.e., mod 𝑁 for some 𝑁, often prime) and the outer argument selects the integer or equivalence class (if you want to think about it that way) from the integers mod 𝑁. In order to ensure the supremum is well-defined, we only define the expression when 𝐴 and 𝑁 are coprime. (Contributed by Mario Carneiro, 23-Feb-2014.) (Revised by AV, 26-Sep-2020.)
Assertion
Ref Expression
odzval ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((od𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
Distinct variable groups:   𝑛,𝑁   𝐴,𝑛

Proof of Theorem odzval
Dummy variables 𝑚 𝑥 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 oveq2 7263 . . . . . . . . 9 (𝑚 = 𝑁 → (𝑥 gcd 𝑚) = (𝑥 gcd 𝑁))
21eqeq1d 2740 . . . . . . . 8 (𝑚 = 𝑁 → ((𝑥 gcd 𝑚) = 1 ↔ (𝑥 gcd 𝑁) = 1))
32rabbidv 3404 . . . . . . 7 (𝑚 = 𝑁 → {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} = {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑁) = 1})
4 oveq1 7262 . . . . . . . . 9 (𝑛 = 𝑥 → (𝑛 gcd 𝑁) = (𝑥 gcd 𝑁))
54eqeq1d 2740 . . . . . . . 8 (𝑛 = 𝑥 → ((𝑛 gcd 𝑁) = 1 ↔ (𝑥 gcd 𝑁) = 1))
65cbvrabv 3416 . . . . . . 7 {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} = {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑁) = 1}
73, 6eqtr4di 2797 . . . . . 6 (𝑚 = 𝑁 → {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} = {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1})
8 breq1 5073 . . . . . . . 8 (𝑚 = 𝑁 → (𝑚 ∥ ((𝑥𝑛) − 1) ↔ 𝑁 ∥ ((𝑥𝑛) − 1)))
98rabbidv 3404 . . . . . . 7 (𝑚 = 𝑁 → {𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)} = {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)})
109infeq1d 9166 . . . . . 6 (𝑚 = 𝑁 → inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < ) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))
117, 10mpteq12dv 5161 . . . . 5 (𝑚 = 𝑁 → (𝑥 ∈ {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
12 df-odz 16394 . . . . 5 od = (𝑚 ∈ ℕ ↦ (𝑥 ∈ {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
13 zex 12258 . . . . . 6 ℤ ∈ V
1413mptrabex 7083 . . . . 5 (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) ∈ V
1511, 12, 14fvmpt 6857 . . . 4 (𝑁 ∈ ℕ → (od𝑁) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
1615fveq1d 6758 . . 3 (𝑁 ∈ ℕ → ((od𝑁)‘𝐴) = ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴))
17 oveq1 7262 . . . . . 6 (𝑛 = 𝐴 → (𝑛 gcd 𝑁) = (𝐴 gcd 𝑁))
1817eqeq1d 2740 . . . . 5 (𝑛 = 𝐴 → ((𝑛 gcd 𝑁) = 1 ↔ (𝐴 gcd 𝑁) = 1))
1918elrab 3617 . . . 4 (𝐴 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↔ (𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1))
20 oveq1 7262 . . . . . . . . 9 (𝑥 = 𝐴 → (𝑥𝑛) = (𝐴𝑛))
2120oveq1d 7270 . . . . . . . 8 (𝑥 = 𝐴 → ((𝑥𝑛) − 1) = ((𝐴𝑛) − 1))
2221breq2d 5082 . . . . . . 7 (𝑥 = 𝐴 → (𝑁 ∥ ((𝑥𝑛) − 1) ↔ 𝑁 ∥ ((𝐴𝑛) − 1)))
2322rabbidv 3404 . . . . . 6 (𝑥 = 𝐴 → {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)} = {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)})
2423infeq1d 9166 . . . . 5 (𝑥 = 𝐴 → inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
25 eqid 2738 . . . . 5 (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))
26 ltso 10986 . . . . . 6 < Or ℝ
2726infex 9182 . . . . 5 inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ) ∈ V
2824, 25, 27fvmpt 6857 . . . 4 (𝐴 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} → ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
2919, 28sylbir 234 . . 3 ((𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
3016, 29sylan9eq 2799 . 2 ((𝑁 ∈ ℕ ∧ (𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1)) → ((od𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
31303impb 1113 1 ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((od𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 395  w3a 1085   = wceq 1539  wcel 2108  {crab 3067   class class class wbr 5070  cmpt 5153  cfv 6418  (class class class)co 7255  infcinf 9130  cr 10801  1c1 10803   < clt 10940  cmin 11135  cn 11903  cz 12249  cexp 13710  cdvds 15891   gcd cgcd 16129  odcodz 16392
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1799  ax-4 1813  ax-5 1914  ax-6 1972  ax-7 2012  ax-8 2110  ax-9 2118  ax-10 2139  ax-11 2156  ax-12 2173  ax-ext 2709  ax-rep 5205  ax-sep 5218  ax-nul 5225  ax-pow 5283  ax-pr 5347  ax-un 7566  ax-cnex 10858  ax-resscn 10859  ax-pre-lttri 10876  ax-pre-lttrn 10877
This theorem depends on definitions:  df-bi 206  df-an 396  df-or 844  df-3or 1086  df-3an 1087  df-tru 1542  df-fal 1552  df-ex 1784  df-nf 1788  df-sb 2069  df-mo 2540  df-eu 2569  df-clab 2716  df-cleq 2730  df-clel 2817  df-nfc 2888  df-ne 2943  df-nel 3049  df-ral 3068  df-rex 3069  df-reu 3070  df-rmo 3071  df-rab 3072  df-v 3424  df-sbc 3712  df-csb 3829  df-dif 3886  df-un 3888  df-in 3890  df-ss 3900  df-nul 4254  df-if 4457  df-pw 4532  df-sn 4559  df-pr 4561  df-op 4565  df-uni 4837  df-iun 4923  df-br 5071  df-opab 5133  df-mpt 5154  df-id 5480  df-po 5494  df-so 5495  df-xp 5586  df-rel 5587  df-cnv 5588  df-co 5589  df-dm 5590  df-rn 5591  df-res 5592  df-ima 5593  df-iota 6376  df-fun 6420  df-fn 6421  df-f 6422  df-f1 6423  df-fo 6424  df-f1o 6425  df-fv 6426  df-ov 7258  df-er 8456  df-en 8692  df-dom 8693  df-sdom 8694  df-sup 9131  df-inf 9132  df-pnf 10942  df-mnf 10943  df-ltxr 10945  df-neg 11138  df-z 12250  df-odz 16394
This theorem is referenced by:  odzcllem  16421  odzdvds  16424
  Copyright terms: Public domain W3C validator