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

Theorem odzval 16118
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 7143 . . . . . . . . 9 (𝑚 = 𝑁 → (𝑥 gcd 𝑚) = (𝑥 gcd 𝑁))
21eqeq1d 2800 . . . . . . . 8 (𝑚 = 𝑁 → ((𝑥 gcd 𝑚) = 1 ↔ (𝑥 gcd 𝑁) = 1))
32rabbidv 3427 . . . . . . 7 (𝑚 = 𝑁 → {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} = {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑁) = 1})
4 oveq1 7142 . . . . . . . . 9 (𝑛 = 𝑥 → (𝑛 gcd 𝑁) = (𝑥 gcd 𝑁))
54eqeq1d 2800 . . . . . . . 8 (𝑛 = 𝑥 → ((𝑛 gcd 𝑁) = 1 ↔ (𝑥 gcd 𝑁) = 1))
65cbvrabv 3439 . . . . . . 7 {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} = {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑁) = 1}
73, 6eqtr4di 2851 . . . . . 6 (𝑚 = 𝑁 → {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} = {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1})
8 breq1 5033 . . . . . . . 8 (𝑚 = 𝑁 → (𝑚 ∥ ((𝑥𝑛) − 1) ↔ 𝑁 ∥ ((𝑥𝑛) − 1)))
98rabbidv 3427 . . . . . . 7 (𝑚 = 𝑁 → {𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)} = {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)})
109infeq1d 8925 . . . . . 6 (𝑚 = 𝑁 → inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < ) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))
117, 10mpteq12dv 5115 . . . . 5 (𝑚 = 𝑁 → (𝑥 ∈ {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
12 df-odz 16092 . . . . 5 od = (𝑚 ∈ ℕ ↦ (𝑥 ∈ {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
13 zex 11978 . . . . . 6 ℤ ∈ V
1413mptrabex 6965 . . . . 5 (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) ∈ V
1511, 12, 14fvmpt 6745 . . . 4 (𝑁 ∈ ℕ → (od𝑁) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
1615fveq1d 6647 . . 3 (𝑁 ∈ ℕ → ((od𝑁)‘𝐴) = ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴))
17 oveq1 7142 . . . . . 6 (𝑛 = 𝐴 → (𝑛 gcd 𝑁) = (𝐴 gcd 𝑁))
1817eqeq1d 2800 . . . . 5 (𝑛 = 𝐴 → ((𝑛 gcd 𝑁) = 1 ↔ (𝐴 gcd 𝑁) = 1))
1918elrab 3628 . . . 4 (𝐴 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↔ (𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1))
20 oveq1 7142 . . . . . . . . 9 (𝑥 = 𝐴 → (𝑥𝑛) = (𝐴𝑛))
2120oveq1d 7150 . . . . . . . 8 (𝑥 = 𝐴 → ((𝑥𝑛) − 1) = ((𝐴𝑛) − 1))
2221breq2d 5042 . . . . . . 7 (𝑥 = 𝐴 → (𝑁 ∥ ((𝑥𝑛) − 1) ↔ 𝑁 ∥ ((𝐴𝑛) − 1)))
2322rabbidv 3427 . . . . . 6 (𝑥 = 𝐴 → {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)} = {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)})
2423infeq1d 8925 . . . . 5 (𝑥 = 𝐴 → inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
25 eqid 2798 . . . . 5 (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))
26 ltso 10710 . . . . . 6 < Or ℝ
2726infex 8941 . . . . 5 inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ) ∈ V
2824, 25, 27fvmpt 6745 . . . 4 (𝐴 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} → ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
2919, 28sylbir 238 . . 3 ((𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
3016, 29sylan9eq 2853 . 2 ((𝑁 ∈ ℕ ∧ (𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1)) → ((od𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
31303impb 1112 1 ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((od𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 399  w3a 1084   = wceq 1538  wcel 2111  {crab 3110   class class class wbr 5030  cmpt 5110  cfv 6324  (class class class)co 7135  infcinf 8889  cr 10525  1c1 10527   < clt 10664  cmin 10859  cn 11625  cz 11969  cexp 13425  cdvds 15599   gcd cgcd 15833  odcodz 16090
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1797  ax-4 1811  ax-5 1911  ax-6 1970  ax-7 2015  ax-8 2113  ax-9 2121  ax-10 2142  ax-11 2158  ax-12 2175  ax-ext 2770  ax-rep 5154  ax-sep 5167  ax-nul 5174  ax-pow 5231  ax-pr 5295  ax-un 7441  ax-cnex 10582  ax-resscn 10583  ax-pre-lttri 10600  ax-pre-lttrn 10601
This theorem depends on definitions:  df-bi 210  df-an 400  df-or 845  df-3or 1085  df-3an 1086  df-tru 1541  df-ex 1782  df-nf 1786  df-sb 2070  df-mo 2598  df-eu 2629  df-clab 2777  df-cleq 2791  df-clel 2870  df-nfc 2938  df-ne 2988  df-nel 3092  df-ral 3111  df-rex 3112  df-reu 3113  df-rmo 3114  df-rab 3115  df-v 3443  df-sbc 3721  df-csb 3829  df-dif 3884  df-un 3886  df-in 3888  df-ss 3898  df-nul 4244  df-if 4426  df-pw 4499  df-sn 4526  df-pr 4528  df-op 4532  df-uni 4801  df-iun 4883  df-br 5031  df-opab 5093  df-mpt 5111  df-id 5425  df-po 5438  df-so 5439  df-xp 5525  df-rel 5526  df-cnv 5527  df-co 5528  df-dm 5529  df-rn 5530  df-res 5531  df-ima 5532  df-iota 6283  df-fun 6326  df-fn 6327  df-f 6328  df-f1 6329  df-fo 6330  df-f1o 6331  df-fv 6332  df-ov 7138  df-er 8272  df-en 8493  df-dom 8494  df-sdom 8495  df-sup 8890  df-inf 8891  df-pnf 10666  df-mnf 10667  df-ltxr 10669  df-neg 10862  df-z 11970  df-odz 16092
This theorem is referenced by:  odzcllem  16119  odzdvds  16122
  Copyright terms: Public domain W3C validator