mathlib documentation

non-mathlib.field_definition

@[class]
structure myfld (f : Type) :
Type
def square (f : Type) [myfld f] :
f → f
Equations
@[simp]
theorem add_comm (f : Type) [myfld f] (x y : f) :
x .+ y = y .+ x
@[simp]
theorem one_mul_simp (f : Type) [myfld f] (x : f) :
@[simp]
theorem add_assoc (f : Type) [myfld f] (x y z : f) :
x .+ y .+ z = x .+ (y .+ z)
@[simp]
theorem mul_comm (f : Type) [myfld f] (x y : f) :
x .* y = y .* x
@[simp]
theorem mul_assoc (f : Type) [myfld f] (x y z : f) :
x .* y .* z = x .* (y .* z)
theorem zero_add (f : Type) [myfld f] (x : f) :
@[simp]
theorem zero_simp (f : Type) [myfld f] (x : f) :
@[simp]
theorem simp_zero (f : Type) [myfld f] (x : f) :
@[simp]
theorem distrib_simp (f : Type) [myfld f] (x y z : f) :
(x .+ y) .* z = x .* z .+ y .* z
@[simp]
theorem distrib_simp_alt (f : Type) [myfld f] (x y z : f) :
x .* (y .+ z) = x .* y .+ x .* z
@[simp]
theorem one_mul (f : Type) [myfld f] (x : f) :
@[simp]
theorem simp_mul_one (f : Type) [myfld f] (x : f) :
@[simp]
theorem add_negate_simp (f : Type) [myfld f] (x : f) :
@[simp]
theorem add_negate_simp_alt (f : Type) [myfld f] (x : f) :
@[simp]
theorem mul_reciprocal (f : Type) [myfld f] (x : f) (proof : x myfld.zero) :
theorem equal_ne_zero (f : Type) [myfld f] (x y : f) :
x = yx myfld.zeroy myfld.zero