Mentions légales du service

Skip to content
Snippets Groups Projects
Commit 75f9e888 authored by MARCHE Claude's avatar MARCHE Claude
Browse files

fix type error in algebra

parent 7efae3f8
No related branches found
No related tags found
No related merge requests found
......@@ -90,15 +90,15 @@ theory Field
axiom Inverse : forall x:t. x <> zero -> x * inv x = one
function (/) (x y : t) : t = x * inv y
lemma assoc_mul_div: forall x y z:real.
lemma assoc_mul_div: forall x y z:t.
(* todo: discard the hypothesis ? *)
z <> zero -> (x*y)/z = x*(y/z)
lemma assoc_div_mul: forall x y z:real.
lemma assoc_div_mul: forall x y z:t.
(* todo: discard the hypothesis ? *)
y <> zero /\ z <> zero -> (x/y)/z = x/(y*z)
lemma assoc_div_div: forall x y z:real.
lemma assoc_div_div: forall x y z:t.
(* todo: discard the hypothesis ? *)
y <> zero /\ z <> zero -> x/(y/z) = (x*z)/y
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment