Search for blocks/addresses/...

Proofgold Address

address
PUWsrtMbayBR51BMHLBrsJ39dM7xg8ojgX4
total
0
mg
-
conjpub
-
current assets
20919../4894a.. bday: 23950 doc published by Pr5Zc..
Definition andand := λ x0 x1 : ο . ∀ x2 : ο . (x0x1x2)x2
Param omegaomega : ι
Param mul_natmul_nat : ιιι
Param ordsuccordsucc : ιι
Definition even_nateven_nat := λ x0 . and (x0omega) (∀ x1 : ο . (∀ x2 . and (x2omega) (x0 = mul_nat 2 x2)x1)x1)
Definition FalseFalse := ∀ x0 : ο . x0
Definition notnot := λ x0 : ο . x0False
Definition odd_natodd_nat := λ x0 . and (x0omega) (∀ x1 . x1omegax0 = mul_nat 2 x1∀ x2 : ο . x2)
Known even_nat_not_odd_nateven_nat_not_odd_nat : ∀ x0 . even_nat x0not (odd_nat x0)
Param nat_pnat_p : ιο
Known even_nat_doubleeven_nat_double : ∀ x0 . nat_p x0even_nat (mul_nat 2 x0)
Param exactly1of2exactly1of2 : οοο
Known even_nat_xor_Seven_nat_xor_S : ∀ x0 . nat_p x0exactly1of2 (even_nat x0) (even_nat (ordsucc x0))
Param mul_SNomul_SNo : ιιι
Known mul_nat_mul_SNomul_nat_mul_SNo : ∀ x0 . x0omega∀ x1 . x1omegamul_nat x0 x1 = mul_SNo x0 x1
Known nat_p_omeganat_p_omega : ∀ x0 . nat_p x0x0omega
Known nat_2nat_2 : nat_p 2
Param SNoSNo : ιο
Known mul_SNo_oneLmul_SNo_oneL : ∀ x0 . SNo x0mul_SNo 1 x0 = x0
Known nat_p_SNonat_p_SNo : ∀ x0 . nat_p x0SNo x0
Param eps_eps_ : ιι
Known eps_1_half_eq3eps_1_half_eq3 : mul_SNo (eps_ 1) 2 = 1
Known mul_SNo_assocmul_SNo_assoc : ∀ x0 x1 x2 . SNo x0SNo x1SNo x2mul_SNo x0 (mul_SNo x1 x2) = mul_SNo (mul_SNo x0 x1) x2
Known SNo_eps_SNo_eps_ : ∀ x0 . x0omegaSNo (eps_ x0)
Known nat_1nat_1 : nat_p 1
Theorem double_nat_canceldouble_nat_cancel : ∀ x0 . nat_p x0∀ x1 . nat_p x1mul_nat 2 x0 = mul_nat 2 x1x0 = x1 (proof)
Known andIandI : ∀ x0 x1 : ο . x0x1and x0 x1
Known nat_0nat_0 : nat_p 0
Known mul_nat_0Rmul_nat_0R : ∀ x0 . mul_nat x0 0 = 0
Theorem even_nat_0even_nat_0 : even_nat 0 (proof)
Definition oror := λ x0 x1 : ο . ∀ x2 : ο . (x0x2)(x1x2)x2
Known nat_indnat_ind : ∀ x0 : ι → ο . x0 0(∀ x1 . nat_p x1x0 x1x0 (ordsucc x1))∀ x1 . nat_p x1x0 x1
Known orILorIL : ∀ x0 x1 : ο . x0or x0 x1
Known orIRorIR : ∀ x0 x1 : ο . x1or x0 x1
Known exactly1of2_Eexactly1of2_E : ∀ x0 x1 : ο . exactly1of2 x0 x1∀ x2 : ο . (x0not x1x2)(not x0x1x2)x2
Known omega_ordsuccomega_ordsucc : ∀ x0 . x0omegaordsucc x0omega
Known FalseEFalseE : False∀ x0 : ο . x0
Theorem even_nat_or_odd_nateven_nat_or_odd_nat : ∀ x0 . nat_p x0or (even_nat x0) (odd_nat x0) (proof)
Theorem not_odd_nat_0not_odd_nat_0 : not (odd_nat 0) (proof)
Known omega_nat_pomega_nat_p : ∀ x0 . x0omeganat_p x0
Known nat_ordsuccnat_ordsucc : ∀ x0 . nat_p x0nat_p (ordsucc x0)
Theorem even_nat_odd_nat_Seven_nat_odd_nat_S : ∀ x0 . even_nat x0odd_nat (ordsucc x0) (proof)
Theorem odd_nat_even_nat_Sodd_nat_even_nat_S : ∀ x0 . odd_nat x0even_nat (ordsucc x0) (proof)
Param add_natadd_nat : ιιι
Known add_nat_0Radd_nat_0R : ∀ x0 . add_nat x0 0 = x0
Known exactly1of2_I2exactly1of2_I2 : ∀ x0 x1 : ο . not x0x1exactly1of2 x0 x1
Known add_nat_SRadd_nat_SR : ∀ x0 x1 . nat_p x1add_nat x0 (ordsucc x1) = ordsucc (add_nat x0 x1)
Known add_nat_padd_nat_p : ∀ x0 . nat_p x0∀ x1 . nat_p x1nat_p (add_nat x0 x1)
Known exactly1of2_I1exactly1of2_I1 : ∀ x0 x1 : ο . x0not x1exactly1of2 x0 x1
Theorem odd_nat_xor_odd_sumodd_nat_xor_odd_sum : ∀ x0 . odd_nat x0∀ x1 . nat_p x1exactly1of2 (odd_nat x1) (odd_nat (add_nat x0 x1)) (proof)
Param iffiff : οοο
Known iff_refliff_refl : ∀ x0 : ο . iff x0 x0
Known mul_nat_SRmul_nat_SR : ∀ x0 x1 . nat_p x1mul_nat x0 (ordsucc x1) = add_nat x0 (mul_nat x0 x1)
Known iffIiffI : ∀ x0 x1 : ο . (x0x1)(x1x0)iff x0 x1
Known mul_nat_pmul_nat_p : ∀ x0 . nat_p x0∀ x1 . nat_p x1nat_p (mul_nat x0 x1)
Known iffERiffER : ∀ x0 x1 : ο . iff x0 x1x1x0
Known iffELiffEL : ∀ x0 x1 : ο . iff x0 x1x0x1
Theorem odd_nat_iff_odd_mul_natodd_nat_iff_odd_mul_nat : ∀ x0 . odd_nat x0∀ x1 . nat_p x1iff (odd_nat x1) (odd_nat (mul_nat x0 x1)) (proof)
Theorem odd_nat_mul_natodd_nat_mul_nat : ∀ x0 x1 . odd_nat x0odd_nat x1odd_nat (mul_nat x0 x1) (proof)
Known nat_invnat_inv : ∀ x0 . nat_p x0or (x0 = 0) (∀ x1 : ο . (∀ x2 . and (nat_p x2) (x0 = ordsucc x2)x1)x1)
Known neq_ordsucc_0neq_ordsucc_0 : ∀ x0 . ordsucc x0 = 0∀ x1 : ο . x1
Known add_nat_SLadd_nat_SL : ∀ x0 . nat_p x0∀ x1 . nat_p x1add_nat (ordsucc x0) x1 = ordsucc (add_nat x0 x1)
Theorem add_nat_0_invadd_nat_0_inv : ∀ x0 . x0omega∀ x1 . x1omegaadd_nat x0 x1 = 0and (x0 = 0) (x1 = 0) (proof)
Theorem mul_nat_0_invmul_nat_0_inv : ∀ x0 . x0omega∀ x1 . x1omegamul_nat x0 x1 = 0or (x0 = 0) (x1 = 0) (proof)
Known mul_nat_1Rmul_nat_1R : ∀ x0 . mul_nat x0 1 = x0
Known In_1_2In_1_2 : 12
Known add_nat_0Ladd_nat_0L : ∀ x0 . nat_p x0add_nat 0 x0 = x0
Param ordinalordinal : ιο
Known ordinal_ordsucc_Inordinal_ordsucc_In : ∀ x0 . ordinal x0∀ x1 . x1x0ordsucc x1ordsucc x0
Known nat_p_ordinalnat_p_ordinal : ∀ x0 . nat_p x0ordinal x0
Definition SubqSubq := λ x0 x1 . ∀ x2 . x2x0x2x1
Known ordsuccI1ordsuccI1 : ∀ x0 . x0ordsucc x0
Theorem ordsucc_in_double_nat_ordsuccordsucc_in_double_nat_ordsucc : ∀ x0 . nat_p x0ordsucc x0mul_nat 2 (ordsucc x0) (proof)
Definition nInnIn := λ x0 x1 . not (x0x1)
Known In_irrefIn_irref : ∀ x0 . nIn x0 x0
Theorem double_nat_Subq_0double_nat_Subq_0 : ∀ x0 . nat_p x0mul_nat 2 x0x0x0 = 0 (proof)
Known Subq_refSubq_ref : ∀ x0 . x0x0
Known Subq_traSubq_tra : ∀ x0 x1 x2 . x0x1x1x2x0x2
Theorem add_nat_Subq_Ladd_nat_Subq_L : ∀ x0 . nat_p x0∀ x1 . nat_p x1x0add_nat x0 x1 (proof)
Known Empty_Subq_eqEmpty_Subq_eq : ∀ x0 . x00x0 = 0
Known ordinal_In_Or_Subqordinal_In_Or_Subq : ∀ x0 x1 . ordinal x0ordinal x1or (x0x1) (x1x0)
Known set_extset_ext : ∀ x0 x1 . x0x1x1x0x0 = x1
Known ordsuccEordsuccE : ∀ x0 x1 . x1ordsucc x0or (x1x0) (x1 = x0)
Known nat_transnat_trans : ∀ x0 . nat_p x0∀ x1 . x1x0x1x0
Known mul_nat_SLmul_nat_SL : ∀ x0 . nat_p x0∀ x1 . nat_p x1mul_nat (ordsucc x0) x1 = add_nat (mul_nat x0 x1) x1
Known add_nat_comadd_nat_com : ∀ x0 . nat_p x0∀ x1 . nat_p x1add_nat x0 x1 = add_nat x1 x0
Theorem square_nat_Subqsquare_nat_Subq : ∀ x0 . nat_p x0∀ x1 . nat_p x1x0x1mul_nat x0 x0mul_nat x1 x1 (proof)
Known nat_complete_indnat_complete_ind : ∀ x0 : ι → ο . (∀ x1 . nat_p x1(∀ x2 . x2x1x0 x2)x0 x1)∀ x1 . nat_p x1x0 x1
Known dnegdneg : ∀ x0 : ο . not (not x0)x0
Known mul_nat_assomul_nat_asso : ∀ x0 . nat_p x0∀ x1 . nat_p x1∀ x2 . nat_p x2mul_nat (mul_nat x0 x1) x2 = mul_nat x0 (mul_nat x1 x2)
Known mul_nat_commul_nat_com : ∀ x0 . nat_p x0∀ x1 . nat_p x1mul_nat x0 x1 = mul_nat x1 x0
Theorem form100_1_v1_lemform100_1_v1_lem : ∀ x0 . nat_p x0∀ x1 . nat_p x1mul_nat x0 x0 = mul_nat 2 (mul_nat x1 x1)x1 = 0 (proof)
Param setminussetminus : ιιι
Known setminusEsetminusE : ∀ x0 x1 x2 . x2setminus x0 x1and (x2x0) (nIn x2 x1)
Known In_0_1In_0_1 : 01
Theorem form100_1_v1form100_1_v1 : ∀ x0 . x0setminus omega 1∀ x1 . x1setminus omega 1mul_nat x0 x0 = mul_nat 2 (mul_nat x1 x1)∀ x2 : ο . x2 (proof)

previous assets