Equations
- fourth_power f a = a .* (a .* (a .* a))
theorem
fourth_power_of_product
(f : Type)
[myfld f]
(a b : f) :
fourth_power f a .* b = (fourth_power f a) .* (fourth_power f b)
Equations
- fourth_root_a f a = sqroot sqroot a
theorem
fourth_root_to_power_a
(f : Type)
[myfld f]
[fld_with_sqrt f]
(a : f) :
fourth_power f (fourth_root_a f a) = a
Equations
- fourth_root_b f a = .- sqroot sqroot a
theorem
fourth_root_to_power_b
(f : Type)
[myfld f]
[fld_with_sqrt f]
(a : f) :
fourth_power f (fourth_root_b f a) = a
Equations
- fourth_root_c f a = sqroot .- sqroot a
theorem
fourth_root_to_power_c
(f : Type)
[myfld f]
[fld_with_sqrt f]
(a : f) :
fourth_power f (fourth_root_c f a) = a
theorem
fourth_root_to_power_d
(f : Type)
[myfld f]
[fld_with_sqrt f]
(a : f) :
fourth_power f (fourth_root_d f a) = a
theorem
multiply_out_fourth_power
(f : Type)
[myfld f]
(x y : f) :
fourth_power f x .+ y = quartic_expression f x myfld.one (four f) .* y (six f) .* (square f y) (four f) .* (cubed f y) (fourth_power f y)
theorem
sum_of_fourth_roots
(f : Type)
[myfld f]
[fld_with_sqrt f]
(x : f) :
(fourth_root_a f x) .+ ((fourth_root_b f x) .+ ((fourth_root_c f x) .+ (fourth_root_d f x))) = myfld.zero
theorem
no_other_fourth_roots
(f : Type)
[myfld f]
[fld_with_sqrt f]
(x root : f) :
root ≠ fourth_root_a f x → root ≠ fourth_root_b f x → root ≠ fourth_root_c f x → root ≠ fourth_root_d f x → fourth_power f root ≠ x
theorem
remove_fourth_power_coefficient
(f : Type)
[myfld f]
(a b c d e x : f)
(a_ne_zero : a ≠ myfld.zero) :
quartic_expression f x a b c d e = myfld.zero ↔ quartic_expression f x myfld.one b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero) = myfld.zero
Equations
- depressed_quartic_subst f c d e x = (fourth_power f x) .+ (c .* (square f x) .+ (d .* x .+ e))
Equations
- pow_of_two f n.succ = (pow_of_two f n) .* (two f)
- pow_of_two f 0 = myfld.one
theorem
pow_of_two_nonzero
(f : Type)
[myfld f]
[fld_not_char_two f]
(exp : ℕ) :
pow_of_two f exp ≠ myfld.zero
Equations
- depressed_quartic_squ_coeff f b c = c .+ .- ((square f b) .* ((three f) .* (myfld.reciprocal (pow_of_two f 3) _)))
Equations
- depressed_quartic_linear_coeff f b c d = (cubed f b) .* (myfld.reciprocal (pow_of_two f 3) _) .+ .- (b .* c .* (myfld.reciprocal (two f) fld_not_char_two.not_char_two)) .+ d
Equations
- depressed_quartic_constant f b c d e = .- ((fourth_power f b) .* ((three f) .* (myfld.reciprocal (pow_of_two f 8) _))) .+ c .* (square f b) .* (myfld.reciprocal (pow_of_two f 4) _) .+ .- (b .* d .* (myfld.reciprocal (four f) _)) .+ e
theorem
quartic_reduce_constant_helper
(f : Type)
[myfld f]
[fld_not_char_two f]
(b c d e : f) :
(fourth_power f .- ((myfld.reciprocal (four f) _) .* b)) .+ ( .- ((cubed f (myfld.reciprocal (four f) _) .* b) .* b) .+ ((myfld.reciprocal (square f (four f)) _) .* ((square f b) .* c) .+ ( .- (b .* ((myfld.reciprocal (four f) _) .* d)) .+ e))) = depressed_quartic_constant f b c d e
theorem
reduce_quartic_to_depressed
(f : Type)
[myfld f]
[fld_not_char_two f]
(b c d e x u : f) :
x = u .+ .- (b .* (myfld.reciprocal (four f) _)) → quartic_expression f x myfld.one b c d e = depressed_quartic_subst f (depressed_quartic_squ_coeff f b c) (depressed_quartic_linear_coeff f b c d) (depressed_quartic_constant f b c d e) u
theorem
depressed_quartic_to_quadratic_product
(f : Type)
[myfld f]
(c d e p q s x : f)
(p_ne_zero : p ≠ myfld.zero) :
theorem
simultaneous_solution_helper
(f : Type)
[myfld f]
[fld_not_char_two f]
(c d e p q s : f)
(p_ne_zero : p ≠ myfld.zero) :
cubic_subst f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) (square f p) = myfld.zero → e = (myfld.reciprocal (two f) .* (two f) _) .* ((fourth_power f p) .+ ((two f) .* (c .* (square f p)) .+ (square f c))) .+ (myfld.reciprocal (two f) .* (two f) _) .* .- (square f d .* (myfld.reciprocal p p_ne_zero))
theorem
simultaneous_solution
(f : Type)
[_inst_1 _inst_2 : myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e p q s : f)
(p_ne_zero : p ≠ myfld.zero)
(int_quantity_ne_zero : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero) :
p = sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero) → s = (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f p) .+ d .* (myfld.reciprocal p p_ne_zero))) → q = (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f p) .+ .- d .* (myfld.reciprocal p p_ne_zero))) → c .+ (square f p) = s .+ q ∧ d .* (myfld.reciprocal p p_ne_zero) = s .+ .- q ∧ e = s .* q
theorem
depressed_quartic_to_quadratic_product_solved
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e x : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
depressed_quartic_subst f c d e x = (quadratic_subst f x myfld.one sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ .- d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _)))) .* (quadratic_subst f x myfld.one .- sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))))
theorem
depressed_quartic_to_linear_factorization
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e x : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
depressed_quartic_subst f c d e x = (x .+ .- (quadratic_formula f myfld.one sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ .- d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one)) .* (x .+ .- (quadratic_formula_alt f myfld.one sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ .- d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one)) .* (x .+ .- (quadratic_formula f myfld.one .- sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one)) .* (x .+ .- (quadratic_formula_alt f myfld.one .- sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one))
theorem
quadratic_product_solution
(f : Type)
[myfld f]
[fld_not_char_two f]
[fld_with_sqrt f]
(b1 b2 c1 c2 x : f) :
x = quadratic_formula f myfld.one b1 c1 myfld.zero_distinct_one ∨ x = quadratic_formula_alt f myfld.one b1 c1 myfld.zero_distinct_one ∨ x = quadratic_formula f myfld.one b2 c2 myfld.zero_distinct_one ∨ x = quadratic_formula_alt f myfld.one b2 c2 myfld.zero_distinct_one → (quadratic_subst f x myfld.one b1 c1) .* (quadratic_subst f x myfld.one b2 c2) = myfld.zero
theorem
quadratic_product_solution_unique
(f : Type)
[myfld f]
[fld_not_char_two f]
[fld_with_sqrt f]
(b1 b2 c1 c2 x : f) :
x ≠ quadratic_formula f myfld.one b1 c1 myfld.zero_distinct_one → x ≠ quadratic_formula_alt f myfld.one b1 c1 myfld.zero_distinct_one → x ≠ quadratic_formula f myfld.one b2 c2 myfld.zero_distinct_one → x ≠ quadratic_formula_alt f myfld.one b2 c2 myfld.zero_distinct_one → (quadratic_subst f x myfld.one b1 c1) .* (quadratic_subst f x myfld.one b2 c2) ≠ myfld.zero
def
depressed_quartic_solution_a
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- depressed_quartic_solution_a f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = quadratic_formula f myfld.one sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ .- d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one
theorem
depressed_quartic_solution_a_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
depressed_quartic_subst f c d e (depressed_quartic_solution_a f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) = myfld.zero
def
depressed_quartic_solution_b
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- depressed_quartic_solution_b f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = quadratic_formula_alt f myfld.one sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ .- d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one
theorem
depressed_quartic_solution_b_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
depressed_quartic_subst f c d e (depressed_quartic_solution_b f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) = myfld.zero
def
depressed_quartic_solution_c
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- depressed_quartic_solution_c f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = quadratic_formula f myfld.one .- sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one
theorem
depressed_quartic_solution_c_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
depressed_quartic_subst f c d e (depressed_quartic_solution_c f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) = myfld.zero
def
depressed_quartic_solution_d
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- depressed_quartic_solution_d f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = quadratic_formula_alt f myfld.one .- sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) (myfld.reciprocal (two f) fld_not_char_two.not_char_two) .* (c .+ ((square f sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a)) .+ d .* (myfld.reciprocal sqroot (cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a) _))) myfld.zero_distinct_one
theorem
depressed_quartic_solution_d_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
depressed_quartic_subst f c d e (depressed_quartic_solution_d f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) = myfld.zero
theorem
depressed_quartic_solution_uniqueness
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(c d e x : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f c) .+ .- ((four f) .* e))) .+ .- (square f (two f) .* c) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* c (square f c) .+ .- ((four f) .* e) .- (square f d) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
x ≠ depressed_quartic_solution_a f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b → x ≠ depressed_quartic_solution_b f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b → x ≠ depressed_quartic_solution_c f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b → x ≠ depressed_quartic_solution_d f c d e int_quantity_ne_zero_a int_quantity_ne_zero_b → depressed_quartic_subst f c d e x ≠ myfld.zero
def
quartic_formula_int_a
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_int_a f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = (depressed_quartic_solution_a f (depressed_quartic_squ_coeff f b c) (depressed_quartic_linear_coeff f b c d) (depressed_quartic_constant f b c d e) int_quantity_ne_zero_a int_quantity_ne_zero_b) .+ .- (b .* (myfld.reciprocal (four f) _))
theorem
quartic_formula_int_a_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_int_a f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) myfld.one b c d e = myfld.zero
def
quartic_formula_a
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_a f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b = quartic_formula_int_a f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero) int_quantity_ne_zero_a int_quantity_ne_zero_b
theorem
quartic_formula_a_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_a f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b) a b c d e = myfld.zero
def
quartic_formula_int_b
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_int_b f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = (depressed_quartic_solution_b f (depressed_quartic_squ_coeff f b c) (depressed_quartic_linear_coeff f b c d) (depressed_quartic_constant f b c d e) int_quantity_ne_zero_a int_quantity_ne_zero_b) .+ .- (b .* (myfld.reciprocal (four f) _))
theorem
quartic_formula_int_b_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_int_b f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) myfld.one b c d e = myfld.zero
def
quartic_formula_b
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_b f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b = quartic_formula_int_b f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero) int_quantity_ne_zero_a int_quantity_ne_zero_b
theorem
quartic_formula_b_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_b f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b) a b c d e = myfld.zero
def
quartic_formula_int_c
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_int_c f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = (depressed_quartic_solution_c f (depressed_quartic_squ_coeff f b c) (depressed_quartic_linear_coeff f b c d) (depressed_quartic_constant f b c d e) int_quantity_ne_zero_a int_quantity_ne_zero_b) .+ .- (b .* (myfld.reciprocal (four f) _))
theorem
quartic_formula_int_c_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_int_c f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) myfld.one b c d e = myfld.zero
def
quartic_formula_c
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_c f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b = quartic_formula_int_c f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero) int_quantity_ne_zero_a int_quantity_ne_zero_b
theorem
quartic_formula_c_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_c f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b) a b c d e = myfld.zero
def
quartic_formula_int_d
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_int_d f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b = (depressed_quartic_solution_d f (depressed_quartic_squ_coeff f b c) (depressed_quartic_linear_coeff f b c d) (depressed_quartic_constant f b c d e) int_quantity_ne_zero_a int_quantity_ne_zero_b) .+ .- (b .* (myfld.reciprocal (four f) _))
theorem
quartic_formula_int_d_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(b c d e : f)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b c)) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b c) (square f (depressed_quartic_squ_coeff f b c)) .+ .- ((four f) .* (depressed_quartic_constant f b c d e)) .- (square f (depressed_quartic_linear_coeff f b c d)) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_int_d f b c d e int_quantity_ne_zero_a int_quantity_ne_zero_b) myfld.one b c d e = myfld.zero
def
quartic_formula_d
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
f
Equations
- quartic_formula_d f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b = quartic_formula_int_d f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero) int_quantity_ne_zero_a int_quantity_ne_zero_b
theorem
quartic_formula_d_works
(f : Type)
[myfld f]
[fld_with_sqrt f]
[fld_with_cube_root f]
[fld_not_char_two f]
[fld_not_char_three f]
(a b c d e : f)
(a_ne_zero : a ≠ myfld.zero)
(int_quantity_ne_zero_a : (three f) .* (myfld.one .* ((square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))))) .+ .- (square f (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) ≠ myfld.zero)
(int_quantity_ne_zero_b : cubic_formula_a f myfld.one (two f) .* (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero)) (square f (depressed_quartic_squ_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero))) .+ .- ((four f) .* (depressed_quartic_constant f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero) e .* (myfld.reciprocal a a_ne_zero))) .- (square f (depressed_quartic_linear_coeff f b .* (myfld.reciprocal a a_ne_zero) c .* (myfld.reciprocal a a_ne_zero) d .* (myfld.reciprocal a a_ne_zero))) myfld.zero_distinct_one int_quantity_ne_zero_a ≠ myfld.zero) :
quartic_expression f (quartic_formula_d f a b c d e a_ne_zero int_quantity_ne_zero_a int_quantity_ne_zero_b) a b c d e = myfld.zero