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

Theorem odzval 16130
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 7166 . . . . . . . . 9 (𝑚 = 𝑁 → (𝑥 gcd 𝑚) = (𝑥 gcd 𝑁))
21eqeq1d 2825 . . . . . . . 8 (𝑚 = 𝑁 → ((𝑥 gcd 𝑚) = 1 ↔ (𝑥 gcd 𝑁) = 1))
32rabbidv 3482 . . . . . . 7 (𝑚 = 𝑁 → {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} = {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑁) = 1})
4 oveq1 7165 . . . . . . . . 9 (𝑛 = 𝑥 → (𝑛 gcd 𝑁) = (𝑥 gcd 𝑁))
54eqeq1d 2825 . . . . . . . 8 (𝑛 = 𝑥 → ((𝑛 gcd 𝑁) = 1 ↔ (𝑥 gcd 𝑁) = 1))
65cbvrabv 3493 . . . . . . 7 {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} = {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑁) = 1}
73, 6syl6eqr 2876 . . . . . 6 (𝑚 = 𝑁 → {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} = {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1})
8 breq1 5071 . . . . . . . 8 (𝑚 = 𝑁 → (𝑚 ∥ ((𝑥𝑛) − 1) ↔ 𝑁 ∥ ((𝑥𝑛) − 1)))
98rabbidv 3482 . . . . . . 7 (𝑚 = 𝑁 → {𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)} = {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)})
109infeq1d 8943 . . . . . 6 (𝑚 = 𝑁 → inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < ) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))
117, 10mpteq12dv 5153 . . . . 5 (𝑚 = 𝑁 → (𝑥 ∈ {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
12 df-odz 16104 . . . . 5 od = (𝑚 ∈ ℕ ↦ (𝑥 ∈ {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑚) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑚 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
13 zex 11993 . . . . . 6 ℤ ∈ V
1413mptrabex 6990 . . . . 5 (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) ∈ V
1511, 12, 14fvmpt 6770 . . . 4 (𝑁 ∈ ℕ → (od𝑁) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )))
1615fveq1d 6674 . . 3 (𝑁 ∈ ℕ → ((od𝑁)‘𝐴) = ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴))
17 oveq1 7165 . . . . . 6 (𝑛 = 𝐴 → (𝑛 gcd 𝑁) = (𝐴 gcd 𝑁))
1817eqeq1d 2825 . . . . 5 (𝑛 = 𝐴 → ((𝑛 gcd 𝑁) = 1 ↔ (𝐴 gcd 𝑁) = 1))
1918elrab 3682 . . . 4 (𝐴 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↔ (𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1))
20 oveq1 7165 . . . . . . . . 9 (𝑥 = 𝐴 → (𝑥𝑛) = (𝐴𝑛))
2120oveq1d 7173 . . . . . . . 8 (𝑥 = 𝐴 → ((𝑥𝑛) − 1) = ((𝐴𝑛) − 1))
2221breq2d 5080 . . . . . . 7 (𝑥 = 𝐴 → (𝑁 ∥ ((𝑥𝑛) − 1) ↔ 𝑁 ∥ ((𝐴𝑛) − 1)))
2322rabbidv 3482 . . . . . 6 (𝑥 = 𝐴 → {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)} = {𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)})
2423infeq1d 8943 . . . . 5 (𝑥 = 𝐴 → inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
25 eqid 2823 . . . . 5 (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < )) = (𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))
26 ltso 10723 . . . . . 6 < Or ℝ
2726infex 8959 . . . . 5 inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ) ∈ V
2824, 25, 27fvmpt 6770 . . . 4 (𝐴 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} → ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
2919, 28sylbir 237 . . 3 ((𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((𝑥 ∈ {𝑛 ∈ ℤ ∣ (𝑛 gcd 𝑁) = 1} ↦ inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝑥𝑛) − 1)}, ℝ, < ))‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
3016, 29sylan9eq 2878 . 2 ((𝑁 ∈ ℕ ∧ (𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1)) → ((od𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
31303impb 1111 1 ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((od𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴𝑛) − 1)}, ℝ, < ))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 398  w3a 1083   = wceq 1537  wcel 2114  {crab 3144   class class class wbr 5068  cmpt 5148  cfv 6357  (class class class)co 7158  infcinf 8907  cr 10538  1c1 10540   < clt 10677  cmin 10872  cn 11640  cz 11984  cexp 13432  cdvds 15609   gcd cgcd 15845  odcodz 16102
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1796  ax-4 1810  ax-5 1911  ax-6 1970  ax-7 2015  ax-8 2116  ax-9 2124  ax-10 2145  ax-11 2161  ax-12 2177  ax-ext 2795  ax-rep 5192  ax-sep 5205  ax-nul 5212  ax-pow 5268  ax-pr 5332  ax-un 7463  ax-cnex 10595  ax-resscn 10596  ax-pre-lttri 10613  ax-pre-lttrn 10614
This theorem depends on definitions:  df-bi 209  df-an 399  df-or 844  df-3or 1084  df-3an 1085  df-tru 1540  df-ex 1781  df-nf 1785  df-sb 2070  df-mo 2622  df-eu 2654  df-clab 2802  df-cleq 2816  df-clel 2895  df-nfc 2965  df-ne 3019  df-nel 3126  df-ral 3145  df-rex 3146  df-reu 3147  df-rmo 3148  df-rab 3149  df-v 3498  df-sbc 3775  df-csb 3886  df-dif 3941  df-un 3943  df-in 3945  df-ss 3954  df-nul 4294  df-if 4470  df-pw 4543  df-sn 4570  df-pr 4572  df-op 4576  df-uni 4841  df-iun 4923  df-br 5069  df-opab 5131  df-mpt 5149  df-id 5462  df-po 5476  df-so 5477  df-xp 5563  df-rel 5564  df-cnv 5565  df-co 5566  df-dm 5567  df-rn 5568  df-res 5569  df-ima 5570  df-iota 6316  df-fun 6359  df-fn 6360  df-f 6361  df-f1 6362  df-fo 6363  df-f1o 6364  df-fv 6365  df-ov 7161  df-er 8291  df-en 8512  df-dom 8513  df-sdom 8514  df-sup 8908  df-inf 8909  df-pnf 10679  df-mnf 10680  df-ltxr 10682  df-neg 10875  df-z 11985  df-odz 16104
This theorem is referenced by:  odzcllem  16131  odzdvds  16134
  Copyright terms: Public domain W3C validator