mathlib documentation

non-mathlib.numbers

def two (f : Type) [myfld f] :
f
Equations
def four (f : Type) [myfld f] :
f
Equations
@[class]
structure fld_not_char_two (f : Type) [myfld f] :
Type
theorem two_ne_zero (f : Type) [myfld f] [fld_not_char_two f] :
theorem two_plus_two (f : Type) [myfld f] :
(two f) .+ (two f) = (two f) .* (two f)
theorem four_ne_zero (f : Type) [myfld f] [fld_not_char_two f] :
def three (f : Type) [myfld f] :
f
Equations
@[class]
structure fld_not_char_three (f : Type) [myfld f] :
Type
def six (f : Type) [myfld f] :
f
Equations
def nine (f : Type) [myfld f] :
f
Equations
theorem nine_ne_zero (f : Type) [myfld f] [fld_not_char_three f] :
def twenty_seven (f : Type) [myfld f] :
f
Equations
theorem three_cubed (f : Type) [myfld f] :
def nine_minus_one (f : Type) [myfld f] :
def one_plus_three (f : Type) [myfld f] :
myfld.one .+ (three f) = (two f) .* (two f)
theorem two_x_div_two (f : Type) [myfld f] [fld_not_char_two f] (a : f) :