Library mathcomp.algebra.ssralg
(* (c) Copyright 2006-2016 Microsoft Corporation and Inria.
Distributed under the terms of CeCILL-B. *)
From HB Require Import structures.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat div seq.
From mathcomp Require Import choice fintype finfun bigop prime binomial.
Distributed under the terms of CeCILL-B. *)
From HB Require Import structures.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat div seq.
From mathcomp Require Import choice fintype finfun bigop prime binomial.
The algebraic part of the Algebraic Hierarchy, as described in
``Packaging mathematical structures'', TPHOLs09, by
Francois Garillot, Georges Gonthier, Assia Mahboubi, Laurence Rideau
This file defines for each Structure (Zmodule, Ring, etc ...) its type,
its packers and its canonical properties :
NB: The documentation is currently being reworked. Main guideline: it
should focus on describing factories (and mixins which are a special case).
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
[comUnitRingType of R] == a comUnitRingType structure for R created by
merging canonical comRingType and unitRingType
structures on R.
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
List of factories (to use with HB.instance Definition _ := )
TODO : Adding documentation for substructures
In addition to this structure hierarchy, we also develop a separate,
parallel hierarchy for morphisms linking these structures:
Zmodule (additive abelian groups):
zmodType == interface type for Zmodule structure. ZmodType V m == packs the mixin m to build a Zmodule of type zmodType. The carrier type V must have a choiceType canonical structure. [zmodType of V for S] == V-clone of the zmodType structure S: a copy of S where the sort carrier has been replaced by V, and which is therefore a zmodType structure on V. The sort carrier for S must be convertible to V. [zmodType of V] == clone of a canonical zmodType structure on V. Similar to the above, except S is inferred, but possibly with a syntactically different carrier. 0 == the zero (additive identity) of a Zmodule. x + y == the sum of x and y (in a Zmodule).- x == the opposite (additive inverse) of x.
- IsZmodule.Build T addA addC add0x addNx Requires a choiceType on T and declares a Zmodule on T from the algebraic properties of its operations. NB: we have removed the notation ZmodMixin and used IsZmodule.Build
- PreZmodule.Build T injf f0 fN fD Requires a choiceType on T and declares a Zmodule on T from an injection into a Zmodule and morphism properties
Ring (non-commutative rings):
ringType == interface type for a Ring structure. RingType R m == packs the ring mixin m into a ringType. R^c == the converse Ring for R: R^c is convertible to R but when R has a canonical ringType structure R^c has the converse one: if x y : R^c, then x * y = (y : R) * (x : R). [ringType of R for S] == R-clone of the ringType structure S. [ringType of R] == clone of a canonical ringType structure on R. 1 == the multiplicative identity element of a Ring. n%:R == the ring image of an n in nat; this is just notation for 1 *+ n, so 1%:R is convertible to 1 and 2%:R to 1 + 1. <number> == <number>%:R with <number> a sequence of digits x * y == the ring product of x and y. \prod<range> e == iterated product for a ring (cf bigop.v). x ^+ n == x to the nth power with n in nat (non-negative), i.e., x * (x * .. (x * x)..) (n factors); x ^+ 1 is thus convertible to x, and x ^+ 2 to x * x. GRing.sign R b := (-1) ^+ b in R : ringType, with b : bool. This is a parsing-only helper notation, to be used for defining more specific instances. GRing.comm x y <-> x and y commute, i.e., x * y = y * x. GRing.lreg x <-> x if left-regular, i.e., *%R x is injective. GRing.rreg x <-> x if right-regular, i.e., *%R x is injective. [char R] == the characteristic of R, defined as the set of prime numbers p such that p%:R = 0 in R. The set [char R] has at most one element, and is implemented as a pred_nat collective predicate (see prime.v); thus the statement p \in [char R] can be read as `R has characteristic p', while [char R] =i pred0 means `R has characteristic 0' when R is a field. Frobenius_aut chRp == the Frobenius automorphism mapping x in R to x ^+ p, where chRp : p \in [char R] is a proof that R has (non-zero) characteristic p. mulr_closed S <-> collective predicate S is closed under finite products (1 and x * y in S for x, y in S). smulr_closed S <-> collective predicate S is closed under products and opposite (-1 and x * y in S for x, y in S). semiring_closed S <-> collective predicate S is closed under semiring operations (0, 1, x + y and x * y in S). subring_closed S <-> collective predicate S is closed under ring operations (1, x - y and x * y in S). MulrPred mulS == packs mulS : mulr_closed S into a mulrPred S, SmulrPred mulS smulrPred S, semiringPred S, or subringPred S SemiringPred mulS interface structure, corresponding to the above SubRingPred mulS properties, respectively, provided S already has the supplementary zmodType closure properties. The properties above coerce to subproperties so, e.g., ringS : subring_closed S can be used for the proof obligations of all prerequisites. [ringMixin of R by <: ] == ringType mixin for a subType whose base type is a ringType and whose predicate's canonical key is a SubringPred. > As for zmodType predicates, Import DefaultKeying GRing.DefaultPred turns unresolved GRing.Pred unification constraints into proof obligations for basic closure assumptions.- Zmodule_isRing.Build T mulA mul1x mulx1 mulDx mulxD nonzero1 Requires a Zmodule on T and declares a ring on T using the algebraic properties of its multiplicative operators NB: we have removed the notation RingMixin and used Zmodule_isRing.Build instead
- IsRing.Build zero opp add one mul addrA addrC add0r addNr mulrA mul1r
mulr1 mulrDl mulrDr oner_neq0
Requires a choiceType on T and declares a ringType on T from the
properties of the additive and multiplicative operators
- PreRing.Build T injf f1 fM
Requires a zmodType on T and declares a ringType on T from an
injection into a ringType and morphism properties
- PreRing.Build T injf f1 fM
Requires a zmodType on T and declares a ringType on T from an
injection into a ringType and morphism properties
- Ring_hasCommutativeMul.Build T mulC Requires a ringType on T and declares a comRingType on T from the commutativity of the multiplication.
- Zmodule_isComRing.Build T mulA mulC mul1x mulDl nonzero1
Requires a zmodType on T and declares a comRingType on T
from the algebraic properties of the multiplication.
NB: replacement for ComRingMixin that used to construct only a ring
- PreComRing.Build T injf f1 fM
Requires a ringType on T and declares a comRingType on T from an
injection into a comRingType and morphism properties
- PreComRing.Build T injf f1 fM
Requires a ringType on T and declares a comRingType on T from an
injection into a comRingType and morphism properties
- Ring_hasMulInverse R unit inv mulVr divrr unitrP invr_out
Requires a ring on R and declares a unitRing on R using the properties
of the inverse operation and the boolean test for being a unit
(invertible). The inverse of a non-unit x is constrained to be x
x itself (property invr_out)
NB: replaces "UnitRingMixin mulVr mulrV unitP inv0id"
- PreUnitRing.Build R injf fM fV
Requires a ringType on R and declares a unitRingType on R from an
injection into a unitRingType and morphism properties
- PreUnitRing.Build R injf fM fV
Requires a ringType on R and declares a unitRingType on R from an
injection into a unitRingType and morphism properties
- ComRing_hasMulInverse.Build T mulVp intro_unit inv_out Requires a comRingType on T and declares a comUnitRingType on T from algebraic properties of the inverse
IntegralDomain (integral, commutative, ring with partial inverses):
idomainType == interface type for the IntegralDomain structure. IdomainType R mulf_eq0 == packs the integrality property into an idomainType integral domain structure; R must have a comUnitRingType canonical structure. [idomainType of R for S] == R-clone of the idomainType structure S. [idomainType of R] == clone of a canonical idomainType structure on R. [idomainMixin of R by <: ] == mixin axiom for a idomain subType.- ComUnitRing_isIntegral.Build T idomAxiom
Requires a comUnitRingType on T and declares an integral idomainType
on T from the property of no nonzero zero-divisors
- IsField.Build R fieldP Requires a unitRingType on R and declares a fieldType on R from the field axiom (every non-zero is a unit).
- ComRing_isField.Build R mulVf invr0
Requires a comRingType on R and declares a fieldType on R from the
algeraic properties of the inverse
- Field_isDec.Build F satP Requires a FieldType and on R and declares a decFieldType on F from the decidable satifiability theory axiom
- decidable_of_QE.build F wf_proj ok_proj Requires a FieldType on F and declares a decFieldType on F from the properties of a quantifier elimination projection function.
ClosedField (algebraically closed fields):
closedFieldType == interface type for the ClosedField structure. ClosedFieldType F m == packs the closed field mixin m into a closedFieldType. The carrier F must have a decFieldType structure. [closedFieldType of F on S] == F-clone of a closedFieldType structure S. [closedFieldType of F] == clone of a canonicalclosedFieldType structure on F.- Field_isAlgClosed.Build F Requires a FieldType on F and declares a closedFieldType on F from the closure property.
Lmodule (module with left multiplication by external scalars).
lmodType R == interface type for an Lmodule structure with scalars of type R; R must have a ringType structure. LmodMixin scalA scal1v scalxD scalDv == builds an Lmodule mixin from the algebraic properties of the scaling operation; the module carrier type must have a zmodType structure, and the scalar carrier must have a ringType structure. [TODO: is this still up-to-date? ]- Zmodule_isLmodule.Build R T scalA scal1x scalDr scalDl builds
Requires a ringType on R and a Zmodule on T and declares an Lmodule on
R T from the algebraic properties of the
- PreLmodule.Build R T injf fZ
Requires a ringType on R and a Zmodule on T and
declares a lmodType on R T from an
injection into a lmodType and morphism properties
- PreLmodule.Build R T injf fZ
Requires a ringType on R and a Zmodule on T and
declares a lmodType on R T from an
injection into a lmodType and morphism properties
Lalgebra (left algebra, ring with scaling that associates on the left):
lalgType R == interface type for Lalgebra structures with scalars in R; R must have ringType structure. LalgType R V scalAl == packs scalAl : k (x y) = (k x) y into an Lalgebra of type lalgType R. The carrier type V must have both lmodType R and ringType canonical structures.- Lmodule_isLalgebra.Build R T scalAl
Requires a ringType on R and on T, and an Lmodule on R T and declares
an Lalgebra on R T from the associativity of scaling
- PreLalgebra.Build R T injf fM fZ
Requires a ringType on T and and a Lmodule on R T and declares a
lalgType on R T from an
injection into a lalgType and morphism properties
- PreLalgebra.Build R T injf fM fZ
Requires a ringType on T and and a Lmodule on R T and declares a
lalgType on R T from an
injection into a lalgType and morphism properties
Algebra (ring with scaling that associates both left and right):
algType R == type for Algebra structure with scalars in R. R should be a commutative ring. AlgType R A scalAr == packs scalAr : k (x y) = x (k y) into an Algebra Structure of type algType R. The carrier type A must have an lalgType R structure. CommAlgType R A == creates an Algebra structure for an A that has both lalgType R and comRingType structures. [algType R of V for S] == V-clone of an algType R structure on S. [algType R of V] == clone of a canonical algType R structure on V. [algMixin of V by <: ] == mixin axiom for a subType of an algType.- Lalgebra_isAlgebra R V scalrAr
Requires a ringType on R and an Lalgebra on R V, and declares an
algebra on R V using an algebraic property of the scalar operation
Requires a ringType on T and declares a lalgType on R T from an
injection into a lalgType and morphism properties
- Prealgebra.Build R V injf fM fZ
Requires a ringType on R and declares a algType on R V from an
injection into an algType and morphism properties
- Prealgebra.Build R V injf fM fZ
Requires a ringType on R and declares a algType on R V from an
injection into an algType and morphism properties
- is_ComAlgebra.Build R T
Requires a comRing on T and an Lalgebra on R T, and declares a
commutative algebra on R T
Additive (additive functions):
additive f <-> f of type U -> V is additive, i.e., f maps the Zmodule structure of U to that of V, 0 to 0,- to - and + to + (equivalently, binary - to -).
RMorphism (ring morphisms):
multiplicative f <-> f of type R -> S is multiplicative, i.e., f maps 1 and * in R to 1 and * in S, respectively, R ans S must have canonical ringType structures. rmorphism f <-> f is a ring morphism, i.e., f is both additive and multiplicative. {rmorphism R -> S} == the interface type for ring morphisms, i.e., a Structure that encapsulates the rmorphism property for functions f : R -> S; both R and S must have ringType structures. RMorphism morph_f == packs morph_f : rmorphism f into a Ring morphism structure of type {rmorphism R -> S}. AddRMorphism mul_f == packs mul_f : multiplicative f into an rmorphism structure of type {rmorphism R -> S}; f must already have an {additive R -> S} structure. [rmorphism of f as g] == an f-clone of the rmorphism structure of g. [rmorphism of f] == a clone of an existing additive structure on f.- > If R and S are UnitRings the f also maps units to units and inverses of units to inverses; if R is a field then f is a field isomorphism between R and its image.
- > As rmorphism coerces to both additive and multiplicative, all structures for f can be built from a single proof of rmorphism f.
- > Additive properties (raddf_suffix, see below) are duplicated and specialised for RMorphism (as rmorph_suffix). This allows more precise rewriting and cleaner chaining: although raddf lemmas will recognize RMorphism functions, the converse will not hold (we cannot add reverse inheritance rules because of incomplete backtracking in the Canonical Projection unification), so one would have to insert a /= every time one switched from additive to multiplicative rules.
- > The property duplication also means that it is not strictly necessary to declare all Additive instances.
Linear (linear functions):
scalable f <-> f of type U -> V is scalable, i.e., f morphs scaling on U to scaling on V, a *: _ to a *: _. U and V must both have lmodType R structures, for the same ringType R. scalable_for s f <-> f is scalable for scaling operator s, i.e., f morphs a *: _ to s a _; the range of f only need to be a zmodType. The scaling operator s should be one of *:%R (see scalable, above), *%R or a combination nu \; *%R or nu \; *:%R with nu : {rmorphism _}; otherwise some of the theory (e.g., the linearZ rule) will not apply. linear f <-> f of type U -> V is linear, i.e., f morphs linear combinations a *: u + v in U to similar linear combinations in V; U and V must both have lmodType R structures, for the same ringType R. := forall a, {morph f: u v / a *: u + v}. scalar f <-> f of type U -> R is a scalar function, i.e., f (a *: u + v) = a * f u + f v. linear_for s f <-> f is linear for the scaling operator s, i.e., f (a *: u + v) = s a (f u) + f v. The range of f only needs to be a zmodType, but s MUST be of the form described in in scalable_for paragraph for this predicate to type check. lmorphism f <-> f is both additive and scalable. This is in fact equivalent to linear f, although somewhat less convenient to prove. lmorphism_for s f <-> f is both additive and scalable for s. {linear U -> V} == the interface type for linear functions, i.e., a Structure that encapsulates the linear property for functions f : U -> V; both U and V must have lmodType R structures, for the same R. {scalar U} == the interface type for scalar functions, of type U -> R where U has an lmodType R structure. {linear U -> V | s} == the interface type for functions linear for s. Linear lin_f == packs lin_f : lmorphism_for s f into a linear function structure of type {linear U -> V | s}. As linear_for s f coerces to lmorphism_for s f, Linear can be used with lin_f : linear_for s f (indeed, that is the recommended usage). Note that as linear f, scalar f, {linear U -> V} and {scalar U} are simply notation for corresponding generic "_for" forms, Linear can be used for any of these special cases, transparently. AddLinear scal_f == packs scal_f : scalable_for s f into a {linear U -> V | s} structure; f must already have an additive structure; as with Linear, AddLinear can be used with lin_f : linear f, etc [linear of f as g] == an f-clone of the linear structure of g. [linear of f] == a clone of an existing linear structure on f. (a *: u)%Rlin == transient forms that simplify to a *: u, a * u, (a * u)%Rlin nu a *: u, and nu a * u, respectively, and are (a *:^nu u)%Rlin created by rewriting with the linearZ lemma. The (a *^nu u)%Rlin forms allows the RHS of linearZ to be matched reliably, using the GRing.Scale.law structure.- > Similarly to Ring morphisms, additive properties are specialized for linear functions.
- > Although {scalar U} is convertible to {linear U -> R^o}, it does not actually use R^o, so that rewriting preserves the canonical structure of the range of scalar functions.
- > The generic linearZ lemma uses a set of bespoke interface structures to ensure that both left-to-right and right-to-left rewriting work even in the presence of scaling functions that simplify non-trivially (e.g., idfun \; *%R). Because most of the canonical instances and projections are coercions the machinery will be mostly invisible (with only the {linear ...} structure and %Rlin notations showing), but users should beware that in (a *: f u)%Rlin, a actually occurs in the f u subterm.
- > The simpler linear_LR, or more specialized linearZZ and scalarZ rules should be used instead of linearZ if there are complexity issues, as well as for explicit forward and backward application, as the main parameter of linearZ is a proper sub-interface of {linear fUV | s}.
LRMorphism (linear ring morphisms, i.e., algebra morphisms):
lrmorphism f <-> f of type A -> B is a linear Ring (Algebra) morphism: f is both additive, multiplicative and scalable. A and B must both have lalgType R canonical structures, for the same ringType R. lrmorphism_for s f <-> f a linear Ring morphism for the scaling operator s: f is additive, multiplicative and scalable for s. A must be an lalgType R, but B only needs to have a ringType structure. {lrmorphism A -> B} == the interface type for linear morphisms, i.e., a Structure that encapsulates the lrmorphism property for functions f : A -> B; both A and B must have lalgType R structures, for the same R. {lrmorphism A -> B | s} == the interface type for morphisms linear for s. LRmorphism lrmorph_f == packs lrmorph_f : lrmorphism_for s f into a linear morphism structure of type {lrmorphism A -> B | s}. Like Linear, LRmorphism can be used transparently for lrmorphism f. AddLRmorphism scal_f == packs scal_f : scalable_for s f into a linear morphism structure of type {lrmorphism A -> B | s}; f must already have an {rmorphism A -> B} structure, and AddLRmorphism can be applied to a linear_for s f, linear f, scalar f, etc argument, like AddLinear. [lrmorphism of f] == creates an lrmorphism structure from existing rmorphism and linear structures on f; this is the preferred way of creating lrmorphism structures.- > Linear and rmorphism properties do not need to be specialized for as we supply inheritance join instances in both directions.
Set Implicit Arguments.
Declare Scope ring_scope.
Declare Scope term_scope.
Declare Scope linear_ring_scope.
Reserved Notation "+%R" (at level 0).
Reserved Notation "-%R" (at level 0).
Reserved Notation "*%R" (at level 0, format " *%R").
Reserved Notation "*:%R" (at level 0, format " *:%R").
Reserved Notation "n %:R" (at level 2, left associativity, format "n %:R").
Reserved Notation "k %:A" (at level 2, left associativity, format "k %:A").
Reserved Notation "[ 'char' F ]" (at level 0, format "[ 'char' F ]").
Reserved Notation "x %:T" (at level 2, left associativity, format "x %:T").
Reserved Notation "''X_' i" (at level 8, i at level 2, format "''X_' i").
Patch for recurring Coq parser bug: Coq seg faults when a level 200
notation is used as a pattern.
Reserved Notation "''exists' ''X_' i , f"
(at level 199, i at level 2, right associativity,
format "'[hv' ''exists' ''X_' i , '/ ' f ']'").
Reserved Notation "''forall' ''X_' i , f"
(at level 199, i at level 2, right associativity,
format "'[hv' ''forall' ''X_' i , '/ ' f ']'").
Reserved Notation "x ^f" (at level 2, left associativity, format "x ^f").
Reserved Notation "\0" (at level 0).
Reserved Notation "f \+ g" (at level 50, left associativity).
Reserved Notation "f \- g" (at level 50, left associativity).
Reserved Notation "\- f" (at level 35, f at level 35).
Reserved Notation "a \*o f" (at level 40).
Reserved Notation "a \o* f" (at level 40).
Reserved Notation "a \*: f" (at level 40).
Reserved Notation "f \* g" (at level 40, left associativity).
Declare Scope ring_scope.
Delimit Scope ring_scope with R.
Declare Scope term_scope.
Delimit Scope term_scope with T.
Local Open Scope ring_scope.
Module Import GRing.
Import Monoid.Theory.
#[short(type="zmodType")]
HB.structure Definition Zmodule := {V of isZmodule V & Choice V}.
Module ZmodExports.
Bind Scope ring_scope with Zmodule.sort.
#[deprecated(since="mathcomp 2.0.0", note="use GRing.isZmodule.Build instead")]
Notation ZmodMixin V := (isZmodule.Build V).
Notation "[ 'zmodType' 'of' T 'for' cT ]" := (@Zmodule.clone T%type cT)
(at level 0, format "[ 'zmodType' 'of' T 'for' cT ]") : form_scope.
Notation "[ 'zmodType' 'of' T ]" := (@Zmodule.clone T%type _)
(at level 0, format "[ 'zmodType' 'of' T ]") : form_scope.
End ZmodExports.
Definition natmul V x n := nosimpl iterop _ n +%R x (@zero V).
Section ZmoduleTheory.
Variable V : zmodType.
Implicit Types x y : V.
Lemma addr0 : @right_id V V 0 +%R.
Lemma addrN : @right_inverse V V V 0 -%R +%R.
Definition subrr := addrN.
#[export]
HB.instance Definition _ := Monoid.isComLaw.Build V 0 +%R addrA addrC add0r.
Lemma addrCA : @left_commutative V V +%R.
Lemma addrAC : @right_commutative V V +%R.
Lemma addrACA : @interchange V +%R +%R.
Lemma addKr : @left_loop V V -%R +%R.
Lemma addNKr : @rev_left_loop V V -%R +%R.
Lemma addrK : @right_loop V V -%R +%R.
Lemma addrNK : @rev_right_loop V V -%R +%R.
Definition subrK := addrNK.
Lemma subKr x : involutive (fun y ⇒ x - y).
Lemma addrI : @right_injective V V V +%R.
Lemma addIr : @left_injective V V V +%R.
Lemma subrI : right_injective (fun x y ⇒ x - y).
Lemma subIr : left_injective (fun x y ⇒ x - y).
Lemma opprK : @involutive V -%R.
Lemma oppr_inj : @injective V V -%R.
Lemma oppr0 : -0 = 0 :> V.
Lemma oppr_eq0 x : (- x == 0) = (x == 0).
Lemma subr0 x : x - 0 = x.
Lemma sub0r x : 0 - x = - x.
Lemma opprB x y : - (x - y) = y - x.
Lemma opprD : {morph -%R: x y / x + y : V}.
Lemma addrKA z x y : (x + z) - (z + y) = x - y.
Lemma subrKA z x y : (x - z) + (z + y) = x + y.
Lemma addr0_eq x y : x + y = 0 → - x = y.
Lemma subr0_eq x y : x - y = 0 → x = y.
Lemma subr_eq x y z : (x - z == y) = (x == y + z).
Lemma subr_eq0 x y : (x - y == 0) = (x == y).
Lemma addr_eq0 x y : (x + y == 0) = (x == - y).
Lemma eqr_opp x y : (- x == - y) = (x == y).
Lemma eqr_oppLR x y : (- x == y) = (x == - y).
Lemma mulr0n x : x *+ 0 = 0.
Lemma mulr1n x : x *+ 1 = x.
Lemma mulr2n x : x *+ 2 = x + x.
Lemma mulrS x n : x *+ n.+1 = x + x *+ n.
Lemma mulrSr x n : x *+ n.+1 = x *+ n + x.
Lemma mulrb x (b : bool) : x *+ b = (if b then x else 0).
Lemma mul0rn n : 0 *+ n = 0 :> V.
Lemma mulNrn x n : (- x) *+ n = x *- n.
Lemma mulrnDl n : {morph (fun x ⇒ x *+ n) : x y / x + y}.
Lemma mulrnDr x m n : x *+ (m + n) = x *+ m + x *+ n.
Lemma mulrnBl n : {morph (fun x ⇒ x *+ n) : x y / x - y}.
Lemma mulrnBr x m n : n ≤ m → x *+ (m - n) = x *+ m - x *+ n.
Lemma mulrnA x m n : x *+ (m × n) = x *+ m *+ n.
Lemma mulrnAC x m n : x *+ m *+ n = x *+ n *+ m.
Lemma iter_addr n x y : iter n (+%R x) y = x *+ n + y.
Lemma iter_addr_0 n x : iter n (+%R x) 0 = x *+ n.
Lemma sumrN I r P (F : I → V) :
(\sum_(i <- r | P i) - F i = - (\sum_(i <- r | P i) F i)).
Lemma sumrB I r (P : pred I) (F1 F2 : I → V) :
\sum_(i <- r | P i) (F1 i - F2 i)
= \sum_(i <- r | P i) F1 i - \sum_(i <- r | P i) F2 i.
Lemma sumrMnl I r P (F : I → V) n :
\sum_(i <- r | P i) F i *+ n = (\sum_(i <- r | P i) F i) *+ n.
Lemma sumrMnr x I r P (F : I → nat) :
\sum_(i <- r | P i) x *+ F i = x *+ (\sum_(i <- r | P i) F i).
Lemma sumr_const (I : finType) (A : pred I) x : \sum_(i in A) x = x *+ #|A|.
Lemma sumr_const_nat m n x : \sum_(n ≤ i < m) x = x *+ (m - n).
Lemma telescope_sumr n m (f : nat → V) : n ≤ m →
\sum_(n ≤ k < m) (f k.+1 - f k) = f m - f n.
Section ClosedPredicates.
Variable S : {pred V}.
Definition addr_closed := 0 \in S ∧ {in S &, ∀ u v, u + v \in S}.
Definition oppr_closed := {in S, ∀ u, - u \in S}.
Definition subr_2closed := {in S &, ∀ u v, u - v \in S}.
Definition zmod_closed := 0 \in S ∧ subr_2closed.
Lemma zmod_closedN : zmod_closed → oppr_closed.
Lemma zmod_closedD : zmod_closed → addr_closed.
End ClosedPredicates.
End ZmoduleTheory.
Arguments addrI {V} y [x1 x2].
Arguments addIr {V} x [x1 x2].
Arguments opprK {V}.
Arguments oppr_inj {V} [x1 x2].
#[short(type="ringType")]
HB.structure Definition Ring := { R of isRing R & Choice R }.
Module RingExports.
Bind Scope ring_scope with Ring.sort.
Notation "[ 'ringType' 'of' T 'for' cT ]" := (Ring.clone T%type cT)
(at level 0, format "[ 'ringType' 'of' T 'for' cT ]") : form_scope.
Notation "[ 'ringType' 'of' T ]" := (Ring.clone T%type _)
(at level 0, format "[ 'ringType' 'of' T ]") : form_scope.
End RingExports.
Definition exp R x n := nosimpl iterop _ n (@mul R) x (@one R).
Notation sign R b := (exp (- @one R) (nat_of_bool b)) (only parsing).
Definition comm R x y := @mul R x y = mul y x.
Definition lreg R x := injective (@mul R x).
Definition rreg R x := injective ((@mul R)^~ x).
(at level 199, i at level 2, right associativity,
format "'[hv' ''exists' ''X_' i , '/ ' f ']'").
Reserved Notation "''forall' ''X_' i , f"
(at level 199, i at level 2, right associativity,
format "'[hv' ''forall' ''X_' i , '/ ' f ']'").
Reserved Notation "x ^f" (at level 2, left associativity, format "x ^f").
Reserved Notation "\0" (at level 0).
Reserved Notation "f \+ g" (at level 50, left associativity).
Reserved Notation "f \- g" (at level 50, left associativity).
Reserved Notation "\- f" (at level 35, f at level 35).
Reserved Notation "a \*o f" (at level 40).
Reserved Notation "a \o* f" (at level 40).
Reserved Notation "a \*: f" (at level 40).
Reserved Notation "f \* g" (at level 40, left associativity).
Declare Scope ring_scope.
Delimit Scope ring_scope with R.
Declare Scope term_scope.
Delimit Scope term_scope with T.
Local Open Scope ring_scope.
Module Import GRing.
Import Monoid.Theory.
#[short(type="zmodType")]
HB.structure Definition Zmodule := {V of isZmodule V & Choice V}.
Module ZmodExports.
Bind Scope ring_scope with Zmodule.sort.
#[deprecated(since="mathcomp 2.0.0", note="use GRing.isZmodule.Build instead")]
Notation ZmodMixin V := (isZmodule.Build V).
Notation "[ 'zmodType' 'of' T 'for' cT ]" := (@Zmodule.clone T%type cT)
(at level 0, format "[ 'zmodType' 'of' T 'for' cT ]") : form_scope.
Notation "[ 'zmodType' 'of' T ]" := (@Zmodule.clone T%type _)
(at level 0, format "[ 'zmodType' 'of' T ]") : form_scope.
End ZmodExports.
Definition natmul V x n := nosimpl iterop _ n +%R x (@zero V).
Section ZmoduleTheory.
Variable V : zmodType.
Implicit Types x y : V.
Lemma addr0 : @right_id V V 0 +%R.
Lemma addrN : @right_inverse V V V 0 -%R +%R.
Definition subrr := addrN.
#[export]
HB.instance Definition _ := Monoid.isComLaw.Build V 0 +%R addrA addrC add0r.
Lemma addrCA : @left_commutative V V +%R.
Lemma addrAC : @right_commutative V V +%R.
Lemma addrACA : @interchange V +%R +%R.
Lemma addKr : @left_loop V V -%R +%R.
Lemma addNKr : @rev_left_loop V V -%R +%R.
Lemma addrK : @right_loop V V -%R +%R.
Lemma addrNK : @rev_right_loop V V -%R +%R.
Definition subrK := addrNK.
Lemma subKr x : involutive (fun y ⇒ x - y).
Lemma addrI : @right_injective V V V +%R.
Lemma addIr : @left_injective V V V +%R.
Lemma subrI : right_injective (fun x y ⇒ x - y).
Lemma subIr : left_injective (fun x y ⇒ x - y).
Lemma opprK : @involutive V -%R.
Lemma oppr_inj : @injective V V -%R.
Lemma oppr0 : -0 = 0 :> V.
Lemma oppr_eq0 x : (- x == 0) = (x == 0).
Lemma subr0 x : x - 0 = x.
Lemma sub0r x : 0 - x = - x.
Lemma opprB x y : - (x - y) = y - x.
Lemma opprD : {morph -%R: x y / x + y : V}.
Lemma addrKA z x y : (x + z) - (z + y) = x - y.
Lemma subrKA z x y : (x - z) + (z + y) = x + y.
Lemma addr0_eq x y : x + y = 0 → - x = y.
Lemma subr0_eq x y : x - y = 0 → x = y.
Lemma subr_eq x y z : (x - z == y) = (x == y + z).
Lemma subr_eq0 x y : (x - y == 0) = (x == y).
Lemma addr_eq0 x y : (x + y == 0) = (x == - y).
Lemma eqr_opp x y : (- x == - y) = (x == y).
Lemma eqr_oppLR x y : (- x == y) = (x == - y).
Lemma mulr0n x : x *+ 0 = 0.
Lemma mulr1n x : x *+ 1 = x.
Lemma mulr2n x : x *+ 2 = x + x.
Lemma mulrS x n : x *+ n.+1 = x + x *+ n.
Lemma mulrSr x n : x *+ n.+1 = x *+ n + x.
Lemma mulrb x (b : bool) : x *+ b = (if b then x else 0).
Lemma mul0rn n : 0 *+ n = 0 :> V.
Lemma mulNrn x n : (- x) *+ n = x *- n.
Lemma mulrnDl n : {morph (fun x ⇒ x *+ n) : x y / x + y}.
Lemma mulrnDr x m n : x *+ (m + n) = x *+ m + x *+ n.
Lemma mulrnBl n : {morph (fun x ⇒ x *+ n) : x y / x - y}.
Lemma mulrnBr x m n : n ≤ m → x *+ (m - n) = x *+ m - x *+ n.
Lemma mulrnA x m n : x *+ (m × n) = x *+ m *+ n.
Lemma mulrnAC x m n : x *+ m *+ n = x *+ n *+ m.
Lemma iter_addr n x y : iter n (+%R x) y = x *+ n + y.
Lemma iter_addr_0 n x : iter n (+%R x) 0 = x *+ n.
Lemma sumrN I r P (F : I → V) :
(\sum_(i <- r | P i) - F i = - (\sum_(i <- r | P i) F i)).
Lemma sumrB I r (P : pred I) (F1 F2 : I → V) :
\sum_(i <- r | P i) (F1 i - F2 i)
= \sum_(i <- r | P i) F1 i - \sum_(i <- r | P i) F2 i.
Lemma sumrMnl I r P (F : I → V) n :
\sum_(i <- r | P i) F i *+ n = (\sum_(i <- r | P i) F i) *+ n.
Lemma sumrMnr x I r P (F : I → nat) :
\sum_(i <- r | P i) x *+ F i = x *+ (\sum_(i <- r | P i) F i).
Lemma sumr_const (I : finType) (A : pred I) x : \sum_(i in A) x = x *+ #|A|.
Lemma sumr_const_nat m n x : \sum_(n ≤ i < m) x = x *+ (m - n).
Lemma telescope_sumr n m (f : nat → V) : n ≤ m →
\sum_(n ≤ k < m) (f k.+1 - f k) = f m - f n.
Section ClosedPredicates.
Variable S : {pred V}.
Definition addr_closed := 0 \in S ∧ {in S &, ∀ u v, u + v \in S}.
Definition oppr_closed := {in S, ∀ u, - u \in S}.
Definition subr_2closed := {in S &, ∀ u v, u - v \in S}.
Definition zmod_closed := 0 \in S ∧ subr_2closed.
Lemma zmod_closedN : zmod_closed → oppr_closed.
Lemma zmod_closedD : zmod_closed → addr_closed.
End ClosedPredicates.
End ZmoduleTheory.
Arguments addrI {V} y [x1 x2].
Arguments addIr {V} x [x1 x2].
Arguments opprK {V}.
Arguments oppr_inj {V} [x1 x2].
#[short(type="ringType")]
HB.structure Definition Ring := { R of isRing R & Choice R }.
Module RingExports.
Bind Scope ring_scope with Ring.sort.
Notation "[ 'ringType' 'of' T 'for' cT ]" := (Ring.clone T%type cT)
(at level 0, format "[ 'ringType' 'of' T 'for' cT ]") : form_scope.
Notation "[ 'ringType' 'of' T ]" := (Ring.clone T%type _)
(at level 0, format "[ 'ringType' 'of' T ]") : form_scope.
End RingExports.
Definition exp R x n := nosimpl iterop _ n (@mul R) x (@one R).
Notation sign R b := (exp (- @one R) (nat_of_bool b)) (only parsing).
Definition comm R x y := @mul R x y = mul y x.
Definition lreg R x := injective (@mul R x).
Definition rreg R x := injective ((@mul R)^~ x).
The ``field'' characteristic; the definition, and many of the theorems,
has to apply to rings as well; indeed, we need the Frobenius automorphism
results for a non commutative ring in the proof of Gorenstein 2.6.3.
Converse ring tag.
Definition converse R : Type := R.
Section RingTheory.
Variable R : ringType.
Implicit Types x y : R.
Lemma oner_eq0 : (1 == 0 :> R) = false.
Lemma mul0r : @left_zero R R 0 *%R.
Lemma mulr0 : @right_zero R R 0 *%R.
Lemma mulrN x y : x × (- y) = - (x × y).
Lemma mulNr x y : (- x) × y = - (x × y).
Lemma mulrNN x y : (- x) × (- y) = x × y.
Lemma mulN1r x : -1 × x = - x.
Lemma mulrN1 x : x × -1 = - x.
#[export]
HB.instance Definition _ := Monoid.isLaw.Build R 1 *%R mulrA mul1r mulr1.
#[export]
HB.instance Definition _ := Monoid.isMulLaw.Build R 0 *%R mul0r mulr0.
#[export]
HB.instance Definition _ := Monoid.isAddLaw.Build R *%R +%R mulrDl mulrDr.
Lemma mulr_suml I r P (F : I → R) x :
(\sum_(i <- r | P i) F i) × x = \sum_(i <- r | P i) F i × x.
Lemma mulr_sumr I r P (F : I → R) x :
x × (\sum_(i <- r | P i) F i) = \sum_(i <- r | P i) x × F i.
Lemma mulrBl x y z : (y - z) × x = y × x - z × x.
Lemma mulrBr x y z : x × (y - z) = x × y - x × z.
Lemma mulrnAl x y n : (x *+ n) × y = (x × y) *+ n.
Lemma mulrnAr x y n : x × (y *+ n) = (x × y) *+ n.
Lemma mulr_natl x n : n%:R × x = x *+ n.
Lemma mulr_natr x n : x × n%:R = x *+ n.
Lemma natrD m n : (m + n)%:R = m%:R + n%:R :> R.
Lemma natr1 n : n%:R + 1 = n.+1%:R :> R.
Lemma nat1r n : 1 + n%:R = n.+1%:R :> R.
Lemma natrB m n : n ≤ m → (m - n)%:R = m%:R - n%:R :> R.
Definition natr_sum := big_morph (natmul 1) natrD (mulr0n 1).
Lemma natrM m n : (m × n)%:R = m%:R × n%:R :> R.
Lemma expr0 x : x ^+ 0 = 1.
Lemma expr1 x : x ^+ 1 = x.
Lemma expr2 x : x ^+ 2 = x × x.
Lemma exprS x n : x ^+ n.+1 = x × x ^+ n.
Lemma expr0n n : 0 ^+ n = (n == 0%N)%:R :> R.
Lemma expr1n n : 1 ^+ n = 1 :> R.
Lemma exprD x m n : x ^+ (m + n) = x ^+ m × x ^+ n.
Lemma exprSr x n : x ^+ n.+1 = x ^+ n × x.
Lemma expr_sum x (I : Type) (s : seq I) (P : pred I) F :
x ^+ (\sum_(i <- s | P i) F i) = \prod_(i <- s | P i) x ^+ F i :> R.
Lemma commr_sym x y : comm x y → comm y x.
Lemma commr_refl x : comm x x.
Lemma commr0 x : comm x 0.
Lemma commr1 x : comm x 1.
Lemma commrN x y : comm x y → comm x (- y).
Lemma commrN1 x : comm x (-1).
Lemma commrD x y z : comm x y → comm x z → comm x (y + z).
Lemma commrB x y z : comm x y → comm x z → comm x (y - z).
Lemma commr_sum (I : Type) (s : seq I) (P : pred I) (F : I → R) x :
(∀ i, P i → comm x (F i)) → comm x (\sum_(i <- s | P i) F i).
Lemma commrMn x y n : comm x y → comm x (y *+ n).
Lemma commrM x y z : comm x y → comm x z → comm x (y × z).
Lemma commr_prod (I : Type) (s : seq I) (P : pred I) (F : I → R) x :
(∀ i, P i → comm x (F i)) → comm x (\prod_(i <- s | P i) F i).
Lemma commr_nat x n : comm x n%:R.
Lemma commrX x y n : comm x y → comm x (y ^+ n).
Lemma exprMn_comm x y n : comm x y → (x × y) ^+ n = x ^+ n × y ^+ n.
Lemma commr_sign x n : comm x ((-1) ^+ n).
Lemma exprMn_n x m n : (x *+ m) ^+ n = x ^+ n *+ (m ^ n) :> R.
Lemma exprM x m n : x ^+ (m × n) = x ^+ m ^+ n.
Lemma exprAC x m n : (x ^+ m) ^+ n = (x ^+ n) ^+ m.
Lemma expr_mod n x i : x ^+ n = 1 → x ^+ (i %% n) = x ^+ i.
Lemma expr_dvd n x i : x ^+ n = 1 → n %| i → x ^+ i = 1.
Lemma natrX n k : (n ^ k)%:R = n%:R ^+ k :> R.
Lemma signr_odd n : (-1) ^+ (odd n) = (-1) ^+ n :> R.
Lemma signr_eq0 n : ((-1) ^+ n == 0 :> R) = false.
Lemma mulr_sign (b : bool) x : (-1) ^+ b × x = (if b then - x else x).
Lemma signr_addb b1 b2 : (-1) ^+ (b1 (+) b2) = (-1) ^+ b1 × (-1) ^+ b2 :> R.
Lemma signrE (b : bool) : (-1) ^+ b = 1 - b.*2%:R :> R.
Lemma signrN b : (-1) ^+ (~~ b) = - (-1) ^+ b :> R.
Lemma mulr_signM (b1 b2 : bool) x1 x2 :
((-1) ^+ b1 × x1) × ((-1) ^+ b2 × x2) = (-1) ^+ (b1 (+) b2) × (x1 × x2).
Lemma exprNn x n : (- x) ^+ n = (-1) ^+ n × x ^+ n :> R.
Lemma sqrrN x : (- x) ^+ 2 = x ^+ 2.
Lemma sqrr_sign n : ((-1) ^+ n) ^+ 2 = 1 :> R.
Lemma signrMK n : @involutive R ( *%R ((-1) ^+ n)).
Lemma lastr_eq0 (s : seq R) x : x != 0 → (last x s == 0) = (last 1 s == 0).
Lemma mulrI_eq0 x y : lreg x → (x × y == 0) = (y == 0).
Lemma lreg_neq0 x : lreg x → x != 0.
Lemma mulrI0_lreg x : (∀ y, x × y = 0 → y = 0) → lreg x.
Lemma lregN x : lreg x → lreg (- x).
Lemma lreg1 : lreg (1 : R).
Lemma lregM x y : lreg x → lreg y → lreg (x × y).
Lemma lregMl (a b: R) : lreg (a × b) → lreg b.
Lemma rregMr (a b: R) : rreg (a × b) → rreg a.
Lemma lregX x n : lreg x → lreg (x ^+ n).
Lemma lreg_sign n : lreg ((-1) ^+ n : R).
Lemma iter_mulr n x y : iter n ( *%R x) y = x ^+ n × y.
Lemma iter_mulr_1 n x : iter n ( *%R x) 1 = x ^+ n.
Lemma prodr_const (I : finType) (A : pred I) x : \prod_(i in A) x = x ^+ #|A|.
Lemma prodr_const_nat n m x : \prod_(n ≤ i < m) x = x ^+ (m - n).
Lemma prodrXr x I r P (F : I → nat) :
\prod_(i <- r | P i) x ^+ F i = x ^+ (\sum_(i <- r | P i) F i).
Lemma prodrN (I : finType) (A : pred I) (F : I → R) :
\prod_(i in A) - F i = (- 1) ^+ #|A| × \prod_(i in A) F i.
Lemma prodrMn (I : Type) (s : seq I) (P : pred I) (F : I → R) (g : I → nat) :
\prod_(i <- s | P i) (F i *+ g i) =
\prod_(i <- s | P i) (F i) *+ \prod_(i <- s | P i) g i.
Lemma prodrMn_const n (I : finType) (A : pred I) (F : I → R) :
\prod_(i in A) (F i *+ n) = \prod_(i in A) F i *+ n ^ #|A|.
Lemma natr_prod I r P (F : I → nat) :
(\prod_(i <- r | P i) F i)%:R = \prod_(i <- r | P i) (F i)%:R :> R.
Lemma exprDn_comm x y n (cxy : comm x y) :
(x + y) ^+ n = \sum_(i < n.+1) (x ^+ (n - i) × y ^+ i) *+ 'C(n, i).
Lemma exprBn_comm x y n (cxy : comm x y) :
(x - y) ^+ n =
\sum_(i < n.+1) ((-1) ^+ i × x ^+ (n - i) × y ^+ i) *+ 'C(n, i).
Lemma subrXX_comm x y n (cxy : comm x y) :
x ^+ n - y ^+ n = (x - y) × (\sum_(i < n) x ^+ (n.-1 - i) × y ^+ i).
Lemma exprD1n x n : (x + 1) ^+ n = \sum_(i < n.+1) x ^+ i *+ 'C(n, i).
Lemma subrX1 x n : x ^+ n - 1 = (x - 1) × (\sum_(i < n) x ^+ i).
Lemma sqrrD1 x : (x + 1) ^+ 2 = x ^+ 2 + x *+ 2 + 1.
Lemma sqrrB1 x : (x - 1) ^+ 2 = x ^+ 2 - x *+ 2 + 1.
Lemma subr_sqr_1 x : x ^+ 2 - 1 = (x - 1) × (x + 1).
Definition Frobenius_aut p of p \in [char R] := fun x ⇒ x ^+ p.
Section FrobeniusAutomorphism.
Variable p : nat.
Hypothesis charFp : p \in [char R].
Lemma charf0 : p%:R = 0 :> R.
Lemma charf_prime : prime p.
Hint Resolve charf_prime : core.
Lemma mulrn_char x : x *+ p = 0.
Lemma natr_mod_char n : (n %% p)%:R = n%:R :> R.
Lemma dvdn_charf n : (p %| n)%N = (n%:R == 0 :> R).
Lemma charf_eq : [char R] =i (p : nat_pred).
Lemma bin_lt_charf_0 k : 0 < k < p → 'C(p, k)%:R = 0 :> R.
Lemma Frobenius_autE x : x^f = x ^+ p.
Lemma Frobenius_aut0 : 0^f = 0.
Lemma Frobenius_aut1 : 1^f = 1.
Lemma Frobenius_autD_comm x y (cxy : comm x y) : (x + y)^f = x^f + y^f.
Lemma Frobenius_autMn x n : (x *+ n)^f = x^f *+ n.
Lemma Frobenius_aut_nat n : (n%:R)^f = n%:R.
Lemma Frobenius_autM_comm x y : comm x y → (x × y)^f = x^f × y^f.
Lemma Frobenius_autX x n : (x ^+ n)^f = x^f ^+ n.
Lemma Frobenius_autN x : (- x)^f = - x^f.
Lemma Frobenius_autB_comm x y : comm x y → (x - y)^f = x^f - y^f.
End FrobeniusAutomorphism.
Lemma exprNn_char x n : [char R].-nat n → (- x) ^+ n = - (x ^+ n).
Section Char2.
Hypothesis charR2 : 2 \in [char R].
Lemma addrr_char2 x : x + x = 0.
Lemma oppr_char2 x : - x = x.
Lemma subr_char2 x y : x - y = x + y.
Lemma addrK_char2 x : involutive (+%R^~ x).
Lemma addKr_char2 x : involutive (+%R x).
End Char2.
Section ClosedPredicates.
Variable S : {pred R}.
Definition mulr_2closed := {in S &, ∀ u v, u × v \in S}.
Definition mulr_closed := 1 \in S ∧ mulr_2closed.
Definition smulr_closed := -1 \in S ∧ mulr_2closed.
Definition semiring_closed := addr_closed S ∧ mulr_closed.
Definition subring_closed := [/\ 1 \in S, subr_2closed S & mulr_2closed].
Lemma smulr_closedM : smulr_closed → mulr_closed.
Lemma smulr_closedN : smulr_closed → oppr_closed S.
Lemma semiring_closedD : semiring_closed → addr_closed S.
Lemma semiring_closedM : semiring_closed → mulr_closed.
Lemma subring_closedB : subring_closed → zmod_closed S.
Lemma subring_closedM : subring_closed → smulr_closed.
Lemma subring_closed_semi : subring_closed → semiring_closed.
End ClosedPredicates.
End RingTheory.
Module ConverseZmodExports.
Section RightRegular.
Variable R : ringType.
Implicit Types x y : R.
End RightRegular.
End ConverseZmodExports.
Section RightRegular.
Variable R : ringType.
Implicit Types x y : R.
Let Rc := [the ringType of R^c].
Lemma mulIr_eq0 x y : rreg x → (y × x == 0) = (y == 0).
Lemma mulIr0_rreg x : (∀ y, y × x = 0 → y = 0) → rreg x.
Lemma rreg_neq0 x : rreg x → x != 0.
Lemma rregN x : rreg x → rreg (- x).
Lemma rreg1 : rreg (1 : R).
Lemma rregM x y : rreg x → rreg y → rreg (x × y).
Lemma revrX x n : (x : Rc) ^+ n = (x : R) ^+ n.
Lemma rregX x n : rreg x → rreg (x ^+ n).
End RightRegular.
#[infer(R), short(type="lmodType")]
HB.structure Definition Lmodule (R : ringType) :=
{M of Zmodule M & Zmodule_isLmodule R M}.
Module LmodExports.
Bind Scope ring_scope with Lmodule.sort.
Notation "[ 'lmodType' R 'of' T 'for' cT ]" :=
(@Lmodule.clone [the ringType of R] T%type cT)
(at level 0, format "[ 'lmodType' R 'of' T 'for' cT ]") : form_scope.
Notation "[ 'lmodType' R 'of' T ]" := [lmodType R of T%type for _]
(at level 0, format "[ 'lmodType' R 'of' T ]") : form_scope.
End LmodExports.
Section LmoduleTheory.
Variables (R : ringType) (V : lmodType R).
Implicit Types (a b c : R) (u v : V).
Section RingTheory.
Variable R : ringType.
Implicit Types x y : R.
Lemma oner_eq0 : (1 == 0 :> R) = false.
Lemma mul0r : @left_zero R R 0 *%R.
Lemma mulr0 : @right_zero R R 0 *%R.
Lemma mulrN x y : x × (- y) = - (x × y).
Lemma mulNr x y : (- x) × y = - (x × y).
Lemma mulrNN x y : (- x) × (- y) = x × y.
Lemma mulN1r x : -1 × x = - x.
Lemma mulrN1 x : x × -1 = - x.
#[export]
HB.instance Definition _ := Monoid.isLaw.Build R 1 *%R mulrA mul1r mulr1.
#[export]
HB.instance Definition _ := Monoid.isMulLaw.Build R 0 *%R mul0r mulr0.
#[export]
HB.instance Definition _ := Monoid.isAddLaw.Build R *%R +%R mulrDl mulrDr.
Lemma mulr_suml I r P (F : I → R) x :
(\sum_(i <- r | P i) F i) × x = \sum_(i <- r | P i) F i × x.
Lemma mulr_sumr I r P (F : I → R) x :
x × (\sum_(i <- r | P i) F i) = \sum_(i <- r | P i) x × F i.
Lemma mulrBl x y z : (y - z) × x = y × x - z × x.
Lemma mulrBr x y z : x × (y - z) = x × y - x × z.
Lemma mulrnAl x y n : (x *+ n) × y = (x × y) *+ n.
Lemma mulrnAr x y n : x × (y *+ n) = (x × y) *+ n.
Lemma mulr_natl x n : n%:R × x = x *+ n.
Lemma mulr_natr x n : x × n%:R = x *+ n.
Lemma natrD m n : (m + n)%:R = m%:R + n%:R :> R.
Lemma natr1 n : n%:R + 1 = n.+1%:R :> R.
Lemma nat1r n : 1 + n%:R = n.+1%:R :> R.
Lemma natrB m n : n ≤ m → (m - n)%:R = m%:R - n%:R :> R.
Definition natr_sum := big_morph (natmul 1) natrD (mulr0n 1).
Lemma natrM m n : (m × n)%:R = m%:R × n%:R :> R.
Lemma expr0 x : x ^+ 0 = 1.
Lemma expr1 x : x ^+ 1 = x.
Lemma expr2 x : x ^+ 2 = x × x.
Lemma exprS x n : x ^+ n.+1 = x × x ^+ n.
Lemma expr0n n : 0 ^+ n = (n == 0%N)%:R :> R.
Lemma expr1n n : 1 ^+ n = 1 :> R.
Lemma exprD x m n : x ^+ (m + n) = x ^+ m × x ^+ n.
Lemma exprSr x n : x ^+ n.+1 = x ^+ n × x.
Lemma expr_sum x (I : Type) (s : seq I) (P : pred I) F :
x ^+ (\sum_(i <- s | P i) F i) = \prod_(i <- s | P i) x ^+ F i :> R.
Lemma commr_sym x y : comm x y → comm y x.
Lemma commr_refl x : comm x x.
Lemma commr0 x : comm x 0.
Lemma commr1 x : comm x 1.
Lemma commrN x y : comm x y → comm x (- y).
Lemma commrN1 x : comm x (-1).
Lemma commrD x y z : comm x y → comm x z → comm x (y + z).
Lemma commrB x y z : comm x y → comm x z → comm x (y - z).
Lemma commr_sum (I : Type) (s : seq I) (P : pred I) (F : I → R) x :
(∀ i, P i → comm x (F i)) → comm x (\sum_(i <- s | P i) F i).
Lemma commrMn x y n : comm x y → comm x (y *+ n).
Lemma commrM x y z : comm x y → comm x z → comm x (y × z).
Lemma commr_prod (I : Type) (s : seq I) (P : pred I) (F : I → R) x :
(∀ i, P i → comm x (F i)) → comm x (\prod_(i <- s | P i) F i).
Lemma commr_nat x n : comm x n%:R.
Lemma commrX x y n : comm x y → comm x (y ^+ n).
Lemma exprMn_comm x y n : comm x y → (x × y) ^+ n = x ^+ n × y ^+ n.
Lemma commr_sign x n : comm x ((-1) ^+ n).
Lemma exprMn_n x m n : (x *+ m) ^+ n = x ^+ n *+ (m ^ n) :> R.
Lemma exprM x m n : x ^+ (m × n) = x ^+ m ^+ n.
Lemma exprAC x m n : (x ^+ m) ^+ n = (x ^+ n) ^+ m.
Lemma expr_mod n x i : x ^+ n = 1 → x ^+ (i %% n) = x ^+ i.
Lemma expr_dvd n x i : x ^+ n = 1 → n %| i → x ^+ i = 1.
Lemma natrX n k : (n ^ k)%:R = n%:R ^+ k :> R.
Lemma signr_odd n : (-1) ^+ (odd n) = (-1) ^+ n :> R.
Lemma signr_eq0 n : ((-1) ^+ n == 0 :> R) = false.
Lemma mulr_sign (b : bool) x : (-1) ^+ b × x = (if b then - x else x).
Lemma signr_addb b1 b2 : (-1) ^+ (b1 (+) b2) = (-1) ^+ b1 × (-1) ^+ b2 :> R.
Lemma signrE (b : bool) : (-1) ^+ b = 1 - b.*2%:R :> R.
Lemma signrN b : (-1) ^+ (~~ b) = - (-1) ^+ b :> R.
Lemma mulr_signM (b1 b2 : bool) x1 x2 :
((-1) ^+ b1 × x1) × ((-1) ^+ b2 × x2) = (-1) ^+ (b1 (+) b2) × (x1 × x2).
Lemma exprNn x n : (- x) ^+ n = (-1) ^+ n × x ^+ n :> R.
Lemma sqrrN x : (- x) ^+ 2 = x ^+ 2.
Lemma sqrr_sign n : ((-1) ^+ n) ^+ 2 = 1 :> R.
Lemma signrMK n : @involutive R ( *%R ((-1) ^+ n)).
Lemma lastr_eq0 (s : seq R) x : x != 0 → (last x s == 0) = (last 1 s == 0).
Lemma mulrI_eq0 x y : lreg x → (x × y == 0) = (y == 0).
Lemma lreg_neq0 x : lreg x → x != 0.
Lemma mulrI0_lreg x : (∀ y, x × y = 0 → y = 0) → lreg x.
Lemma lregN x : lreg x → lreg (- x).
Lemma lreg1 : lreg (1 : R).
Lemma lregM x y : lreg x → lreg y → lreg (x × y).
Lemma lregMl (a b: R) : lreg (a × b) → lreg b.
Lemma rregMr (a b: R) : rreg (a × b) → rreg a.
Lemma lregX x n : lreg x → lreg (x ^+ n).
Lemma lreg_sign n : lreg ((-1) ^+ n : R).
Lemma iter_mulr n x y : iter n ( *%R x) y = x ^+ n × y.
Lemma iter_mulr_1 n x : iter n ( *%R x) 1 = x ^+ n.
Lemma prodr_const (I : finType) (A : pred I) x : \prod_(i in A) x = x ^+ #|A|.
Lemma prodr_const_nat n m x : \prod_(n ≤ i < m) x = x ^+ (m - n).
Lemma prodrXr x I r P (F : I → nat) :
\prod_(i <- r | P i) x ^+ F i = x ^+ (\sum_(i <- r | P i) F i).
Lemma prodrN (I : finType) (A : pred I) (F : I → R) :
\prod_(i in A) - F i = (- 1) ^+ #|A| × \prod_(i in A) F i.
Lemma prodrMn (I : Type) (s : seq I) (P : pred I) (F : I → R) (g : I → nat) :
\prod_(i <- s | P i) (F i *+ g i) =
\prod_(i <- s | P i) (F i) *+ \prod_(i <- s | P i) g i.
Lemma prodrMn_const n (I : finType) (A : pred I) (F : I → R) :
\prod_(i in A) (F i *+ n) = \prod_(i in A) F i *+ n ^ #|A|.
Lemma natr_prod I r P (F : I → nat) :
(\prod_(i <- r | P i) F i)%:R = \prod_(i <- r | P i) (F i)%:R :> R.
Lemma exprDn_comm x y n (cxy : comm x y) :
(x + y) ^+ n = \sum_(i < n.+1) (x ^+ (n - i) × y ^+ i) *+ 'C(n, i).
Lemma exprBn_comm x y n (cxy : comm x y) :
(x - y) ^+ n =
\sum_(i < n.+1) ((-1) ^+ i × x ^+ (n - i) × y ^+ i) *+ 'C(n, i).
Lemma subrXX_comm x y n (cxy : comm x y) :
x ^+ n - y ^+ n = (x - y) × (\sum_(i < n) x ^+ (n.-1 - i) × y ^+ i).
Lemma exprD1n x n : (x + 1) ^+ n = \sum_(i < n.+1) x ^+ i *+ 'C(n, i).
Lemma subrX1 x n : x ^+ n - 1 = (x - 1) × (\sum_(i < n) x ^+ i).
Lemma sqrrD1 x : (x + 1) ^+ 2 = x ^+ 2 + x *+ 2 + 1.
Lemma sqrrB1 x : (x - 1) ^+ 2 = x ^+ 2 - x *+ 2 + 1.
Lemma subr_sqr_1 x : x ^+ 2 - 1 = (x - 1) × (x + 1).
Definition Frobenius_aut p of p \in [char R] := fun x ⇒ x ^+ p.
Section FrobeniusAutomorphism.
Variable p : nat.
Hypothesis charFp : p \in [char R].
Lemma charf0 : p%:R = 0 :> R.
Lemma charf_prime : prime p.
Hint Resolve charf_prime : core.
Lemma mulrn_char x : x *+ p = 0.
Lemma natr_mod_char n : (n %% p)%:R = n%:R :> R.
Lemma dvdn_charf n : (p %| n)%N = (n%:R == 0 :> R).
Lemma charf_eq : [char R] =i (p : nat_pred).
Lemma bin_lt_charf_0 k : 0 < k < p → 'C(p, k)%:R = 0 :> R.
Lemma Frobenius_autE x : x^f = x ^+ p.
Lemma Frobenius_aut0 : 0^f = 0.
Lemma Frobenius_aut1 : 1^f = 1.
Lemma Frobenius_autD_comm x y (cxy : comm x y) : (x + y)^f = x^f + y^f.
Lemma Frobenius_autMn x n : (x *+ n)^f = x^f *+ n.
Lemma Frobenius_aut_nat n : (n%:R)^f = n%:R.
Lemma Frobenius_autM_comm x y : comm x y → (x × y)^f = x^f × y^f.
Lemma Frobenius_autX x n : (x ^+ n)^f = x^f ^+ n.
Lemma Frobenius_autN x : (- x)^f = - x^f.
Lemma Frobenius_autB_comm x y : comm x y → (x - y)^f = x^f - y^f.
End FrobeniusAutomorphism.
Lemma exprNn_char x n : [char R].-nat n → (- x) ^+ n = - (x ^+ n).
Section Char2.
Hypothesis charR2 : 2 \in [char R].
Lemma addrr_char2 x : x + x = 0.
Lemma oppr_char2 x : - x = x.
Lemma subr_char2 x y : x - y = x + y.
Lemma addrK_char2 x : involutive (+%R^~ x).
Lemma addKr_char2 x : involutive (+%R x).
End Char2.
Section ClosedPredicates.
Variable S : {pred R}.
Definition mulr_2closed := {in S &, ∀ u v, u × v \in S}.
Definition mulr_closed := 1 \in S ∧ mulr_2closed.
Definition smulr_closed := -1 \in S ∧ mulr_2closed.
Definition semiring_closed := addr_closed S ∧ mulr_closed.
Definition subring_closed := [/\ 1 \in S, subr_2closed S & mulr_2closed].
Lemma smulr_closedM : smulr_closed → mulr_closed.
Lemma smulr_closedN : smulr_closed → oppr_closed S.
Lemma semiring_closedD : semiring_closed → addr_closed S.
Lemma semiring_closedM : semiring_closed → mulr_closed.
Lemma subring_closedB : subring_closed → zmod_closed S.
Lemma subring_closedM : subring_closed → smulr_closed.
Lemma subring_closed_semi : subring_closed → semiring_closed.
End ClosedPredicates.
End RingTheory.
Module ConverseZmodExports.
Section RightRegular.
Variable R : ringType.
Implicit Types x y : R.
End RightRegular.
End ConverseZmodExports.
Section RightRegular.
Variable R : ringType.
Implicit Types x y : R.
Let Rc := [the ringType of R^c].
Lemma mulIr_eq0 x y : rreg x → (y × x == 0) = (y == 0).
Lemma mulIr0_rreg x : (∀ y, y × x = 0 → y = 0) → rreg x.
Lemma rreg_neq0 x : rreg x → x != 0.
Lemma rregN x : rreg x → rreg (- x).
Lemma rreg1 : rreg (1 : R).
Lemma rregM x y : rreg x → rreg y → rreg (x × y).
Lemma revrX x n : (x : Rc) ^+ n = (x : R) ^+ n.
Lemma rregX x n : rreg x → rreg (x ^+ n).
End RightRegular.
#[infer(R), short(type="lmodType")]
HB.structure Definition Lmodule (R : ringType) :=
{M of Zmodule M & Zmodule_isLmodule R M}.
Module LmodExports.
Bind Scope ring_scope with Lmodule.sort.
Notation "[ 'lmodType' R 'of' T 'for' cT ]" :=
(@Lmodule.clone [the ringType of R] T%type cT)
(at level 0, format "[ 'lmodType' R 'of' T 'for' cT ]") : form_scope.
Notation "[ 'lmodType' R 'of' T ]" := [lmodType R of T%type for _]
(at level 0, format "[ 'lmodType' R 'of' T ]") : form_scope.
End LmodExports.
Section LmoduleTheory.
Variables (R : ringType) (V : lmodType R).
Implicit Types (a b c : R) (u v : V).
TODO: fix the type for the exported operation
Lemma scalerA a b v : scale a (scale b v) = scale (a × b) v.
Lemma scale0r v : 0 *: v = 0.
Lemma scaler0 a : a *: 0 = 0 :> V.
Lemma scaleNr a v : - a *: v = - (a *: v).
Lemma scaleN1r v : (- 1) *: v = - v.
Lemma scalerN a v : a *: (- v) = - (a *: v).
Lemma scalerBl a b v : (a - b) *: v = a *: v - b *: v.
Lemma scalerBr a u v : a *: (u - v) = a *: u - a *: v.
Lemma scaler_nat n v : n%:R *: v = v *+ n.
Lemma scaler_sign (b : bool) v: (-1) ^+ b *: v = (if b then - v else v).
Lemma signrZK n : @involutive V ( *:%R ((-1) ^+ n)).
Lemma scalerMnl a v n : a *: v *+ n = (a *+ n) *: v.
Lemma scalerMnr a v n : a *: v *+ n = a *: (v *+ n).
Lemma scaler_suml v I r (P : pred I) F :
(\sum_(i <- r | P i) F i) *: v = \sum_(i <- r | P i) F i *: v.
Lemma scaler_sumr a I r (P : pred I) (F : I → V) :
a *: (\sum_(i <- r | P i) F i) = \sum_(i <- r | P i) a *: F i.
Section ClosedPredicates.
Variable S : {pred V}.
Definition scaler_closed := ∀ a, {in S, ∀ v, a *: v \in S}.
Definition linear_closed := ∀ a, {in S &, ∀ u v, a *: u + v \in S}.
Definition submod_closed := 0 \in S ∧ linear_closed.
Lemma linear_closedB : linear_closed → subr_2closed S.
Lemma submod_closedB : submod_closed → zmod_closed S.
Lemma submod_closedZ : submod_closed → scaler_closed.
End ClosedPredicates.
End LmoduleTheory.
#[infer(R), short(type="lalgType")]
HB.structure Definition Lalgebra R :=
{A of Lmodule_isLalgebra R A & Ring A & Lmodule R A}.
Module LalgExports.
Bind Scope ring_scope with Lalgebra.sort.
Notation "[ 'lalgType' R 'of' T 'for' cT ]" :=
(Lalgebra.clone [the ringType of R] T%type cT)
(at level 0, format "[ 'lalgType' R 'of' T 'for' cT ]") : form_scope.
Notation "[ 'lalgType' R 'of' T ]" := [lalgType R of T%type for _]
(at level 0, format "[ 'lalgType' R 'of' T ]") : form_scope.
End LalgExports.
Lemma scale0r v : 0 *: v = 0.
Lemma scaler0 a : a *: 0 = 0 :> V.
Lemma scaleNr a v : - a *: v = - (a *: v).
Lemma scaleN1r v : (- 1) *: v = - v.
Lemma scalerN a v : a *: (- v) = - (a *: v).
Lemma scalerBl a b v : (a - b) *: v = a *: v - b *: v.
Lemma scalerBr a u v : a *: (u - v) = a *: u - a *: v.
Lemma scaler_nat n v : n%:R *: v = v *+ n.
Lemma scaler_sign (b : bool) v: (-1) ^+ b *: v = (if b then - v else v).
Lemma signrZK n : @involutive V ( *:%R ((-1) ^+ n)).
Lemma scalerMnl a v n : a *: v *+ n = (a *+ n) *: v.
Lemma scalerMnr a v n : a *: v *+ n = a *: (v *+ n).
Lemma scaler_suml v I r (P : pred I) F :
(\sum_(i <- r | P i) F i) *: v = \sum_(i <- r | P i) F i *: v.
Lemma scaler_sumr a I r (P : pred I) (F : I → V) :
a *: (\sum_(i <- r | P i) F i) = \sum_(i <- r | P i) a *: F i.
Section ClosedPredicates.
Variable S : {pred V}.
Definition scaler_closed := ∀ a, {in S, ∀ v, a *: v \in S}.
Definition linear_closed := ∀ a, {in S &, ∀ u v, a *: u + v \in S}.
Definition submod_closed := 0 \in S ∧ linear_closed.
Lemma linear_closedB : linear_closed → subr_2closed S.
Lemma submod_closedB : submod_closed → zmod_closed S.
Lemma submod_closedZ : submod_closed → scaler_closed.
End ClosedPredicates.
End LmoduleTheory.
#[infer(R), short(type="lalgType")]
HB.structure Definition Lalgebra R :=
{A of Lmodule_isLalgebra R A & Ring A & Lmodule R A}.
Module LalgExports.
Bind Scope ring_scope with Lalgebra.sort.
Notation "[ 'lalgType' R 'of' T 'for' cT ]" :=
(Lalgebra.clone [the ringType of R] T%type cT)
(at level 0, format "[ 'lalgType' R 'of' T 'for' cT ]") : form_scope.
Notation "[ 'lalgType' R 'of' T ]" := [lalgType R of T%type for _]
(at level 0, format "[ 'lalgType' R 'of' T ]") : form_scope.
End LalgExports.
Scalar injection (see the definition of in_alg A below).
Regular ring algebra tag.
Definition regular R : Type := R.
Module RegularLalgExports.
Section LalgebraTheory.
Variables (R : ringType) (A : lalgType R).
Implicit Types x y : A.
End LalgebraTheory.
End RegularLalgExports.
Section LalgebraTheory.
Variables (R : ringType) (A : lalgType R).
Implicit Types x y : A.
Lemma mulr_algl a x : (a *: 1) × x = a *: x.
Section ClosedPredicates.
Variable S : {pred A}.
Definition subalg_closed := [/\ 1 \in S, linear_closed S & mulr_2closed S].
Lemma subalg_closedZ : subalg_closed → submod_closed S.
Lemma subalg_closedBM : subalg_closed → subring_closed S.
End ClosedPredicates.
End LalgebraTheory.
Module RegularLalgExports.
Section LalgebraTheory.
Variables (R : ringType) (A : lalgType R).
Implicit Types x y : A.
End LalgebraTheory.
End RegularLalgExports.
Section LalgebraTheory.
Variables (R : ringType) (A : lalgType R).
Implicit Types x y : A.
Lemma mulr_algl a x : (a *: 1) × x = a *: x.
Section ClosedPredicates.
Variable S : {pred A}.
Definition subalg_closed := [/\ 1 \in S, linear_closed S & mulr_2closed S].
Lemma subalg_closedZ : subalg_closed → submod_closed S.
Lemma subalg_closedBM : subalg_closed → subring_closed S.
End ClosedPredicates.
End LalgebraTheory.
Morphism hierarchy.
Definition additive (U V : zmodType) (f : U → V) :=
{morph f : x y / x - y}.
#[mathcomp(axiom="additive")]
HB.structure Definition Additive (U V : zmodType) := {f of isAdditive U V f}.
Module AdditiveExports.
Module Additive.
Definition map (U V : zmodType) (phUV : phant (U → V)) := Additive.type U V.
Definition apply (U V : zmodType) (phUV : phant (U → V)) := @Additive.sort U V.
End Additive.
Notation "{ 'additive' fUV }" := (Additive.map (Phant fUV%type))
(at level 0, format "{ 'additive' fUV }") : type_scope.
Notation "[ 'additive' 'of' f 'as' g ]" := (Additive.clone _ _ f%function g)
(at level 0, format "[ 'additive' 'of' f 'as' g ]") : form_scope.
Notation "[ 'additive' 'of' f ]" := (Additive.clone _ _ f%function _)
(at level 0, format "[ 'additive' 'of' f ]") : form_scope.
End AdditiveExports.
Lifted additive operations.
Section LiftedZmod.
Variables (U : Type) (V : zmodType).
Definition null_fun_head (phV : phant V) of U : V := let: Phant := phV in 0.
Definition add_fun (f g : U → V) x := f x + g x.
Definition sub_fun (f g : U → V) x := f x - g x.
Definition opp_fun (f : U → V) x := - f x.
End LiftedZmod.
Variables (U : Type) (V : zmodType).
Definition null_fun_head (phV : phant V) of U : V := let: Phant := phV in 0.
Definition add_fun (f g : U → V) x := f x + g x.
Definition sub_fun (f g : U → V) x := f x - g x.
Definition opp_fun (f : U → V) x := - f x.
End LiftedZmod.
Lifted multiplication.
Section LiftedRing.
Variables (R : ringType) (T : Type).
Implicit Type f : T → R.
Definition mull_fun a f x := a × f x.
Definition mulr_fun a f x := f x × a.
Definition mul_fun f g x := f x × g x.
End LiftedRing.
Variables (R : ringType) (T : Type).
Implicit Type f : T → R.
Definition mull_fun a f x := a × f x.
Definition mulr_fun a f x := f x × a.
Definition mul_fun f g x := f x × g x.
End LiftedRing.
Lifted linear operations.
Section LiftedScale.
Variables (R : ringType) (U : Type) (V : lmodType R) (A : lalgType R).
Definition scale_fun a (f : U → V) x := a *: f x.
Definition in_alg_head (phA : phant A) k : A := let: Phant := phA in k%:A.
End LiftedScale.
Notation null_fun V := (null_fun_head (Phant V)) (only parsing).
Variables (R : ringType) (U : Type) (V : lmodType R) (A : lalgType R).
Definition scale_fun a (f : U → V) x := a *: f x.
Definition in_alg_head (phA : phant A) k : A := let: Phant := phA in k%:A.
End LiftedScale.
Notation null_fun V := (null_fun_head (Phant V)) (only parsing).
The real in_alg notation is declared after GRing.Theory so that at least
in Coq 8.2 it gets precedence when GRing.Theory is not imported.
Arguments add_fun {_ _} f g _ /.
Arguments sub_fun {_ _} f g _ /.
Arguments opp_fun {_ _} f _ /.
Arguments mull_fun {_ _} a f _ /.
Arguments mulr_fun {_ _} a f _ /.
Arguments scale_fun {_ _ _} a f _ /.
Arguments mul_fun {_ _} f g _ /.
Section AdditiveTheory.
Section Properties.
Variables (U V : zmodType) (k : unit) (f : {additive U → V}).
Lemma raddfB : {morph f : x y / x - y}.
Lemma raddf0 : f 0 = 0.
Lemma raddf_eq0 x : injective f → (f x == 0) = (x == 0).
Lemma raddf_inj : (∀ x, f x = 0 → x = 0) → injective f.
Lemma raddfN : {morph f : x / - x}.
Lemma raddfD : {morph f : x y / x + y}.
Lemma raddfMn n : {morph f : x / x *+ n}.
Lemma raddfMNn n : {morph f : x / x *- n}.
Lemma raddf_sum I r (P : pred I) E :
f (\sum_(i <- r | P i) E i) = \sum_(i <- r | P i) f (E i).
Lemma can2_additive f' : cancel f f' → cancel f' f → additive f'.
End Properties.
Section RingProperties.
Variables (R S : ringType) (f : {additive R → S}).
Lemma raddfMnat n x : f (n%:R × x) = n%:R × f x.
Lemma raddfMsign n x : f ((-1) ^+ n × x) = (-1) ^+ n × f x.
Variables (U : lmodType R) (V : lmodType S) (h : {additive U → V}).
Lemma raddfZnat n u : h (n%:R *: u) = n%:R *: h u.
Lemma raddfZsign n u : h ((-1) ^+ n *: u) = (-1) ^+ n *: h u.
End RingProperties.
Section AddFun.
Variables (U V W : zmodType) (f g : {additive V → W}) (h : {additive U → V}).
Fact idfun_is_additive : additive (@idfun U).
#[export]
HB.instance Definition _ := isAdditive.Build U U idfun idfun_is_additive.
Fact comp_is_additive : additive (f \o h).
#[export]
HB.instance Definition _ := isAdditive.Build U W (f \o h) comp_is_additive.
Fact opp_is_additive : additive (-%R : U → U).
#[export]
HB.instance Definition _ := isAdditive.Build U U -%R opp_is_additive.
Fact null_fun_is_additive : additive (\0 : U → V).
#[export]
HB.instance Definition _ := isAdditive.Build U V \0 null_fun_is_additive.
Fact add_fun_is_additive : additive (f \+ g).
#[export]
HB.instance Definition _ := isAdditive.Build V W (f \+ g) add_fun_is_additive.
Fact sub_fun_is_additive : additive (f \- g).
#[export]
HB.instance Definition _ := isAdditive.Build V W (f \- g) sub_fun_is_additive.
Fact opp_fun_is_additive : additive (\- g).
#[export]
HB.instance Definition _ := isAdditive.Build V W (\- g) opp_fun_is_additive.
End AddFun.
Section MulFun.
Variables (R : ringType) (U : zmodType).
Variables (a : R) (f : {additive U → R}).
Fact mull_fun_is_additive : additive (a \*o f).
#[export]
HB.instance Definition _ := isAdditive.Build U R (a \*o f) mull_fun_is_additive.
Fact mulr_fun_is_additive : additive (a \o× f).
#[export]
HB.instance Definition _ := isAdditive.Build U R (a \o× f) mulr_fun_is_additive.
End MulFun.
Section ScaleFun.
Variables (R : ringType) (U : zmodType) (V : lmodType R).
Variables (a : R) (f : {additive U → V}).
#[export]
HB.instance Definition _ := isAdditive.Build V V ( *:%R a) (@scalerBr R V a).
#[export]
HB.instance Definition _ := Additive.copy (a \*: f) (f \; *:%R a).
End ScaleFun.
End AdditiveTheory.
Definition multiplicative (R S : ringType) (f : R → S) : Prop :=
{morph f : x y / x × y}%R × (f 1 = 1).
FIXME: Additive has very strange implicit arguments
(without @, one would have to write Additive R f)
Module RMorphismExports.
Module RMorphism.
Definition map (R S : ringType) (phRS : phant (R → S)) := RMorphism.type R S.
Definition apply (R S : ringType) (phRS : phant (R → S)) := @RMorphism.sort R S.
End RMorphism.
Notation "{ 'rmorphism' fRS }" := (RMorphism.map (Phant fRS%type))
(at level 0, format "{ 'rmorphism' fRS }") : type_scope.
Notation "[ 'rmorphism' 'of' f 'as' g ]" := (RMorphism.clone _ _ f%function g)
(at level 0, format "[ 'rmorphism' 'of' f 'as' g ]") : form_scope.
Notation "[ 'rmorphism' 'of' f ]" := (RMorphism.clone _ _ f%function _)
(at level 0, format "[ 'rmorphism' 'of' f ]") : form_scope.
End RMorphismExports.
Section RmorphismTheory.
Section Properties.
Variables (R S : ringType) (k : unit) (f : {rmorphism R → S}).
Lemma rmorph0 : f 0 = 0.
Lemma rmorphN : {morph f : x / - x}.
Lemma rmorphD : {morph f : x y / x + y}.
Lemma rmorphB : {morph f: x y / x - y}.
Lemma rmorphMn n : {morph f : x / x *+ n}.
Lemma rmorphMNn n : {morph f : x / x *- n}.
Lemma rmorph_sum I r (P : pred I) E :
f (\sum_(i <- r | P i) E i) = \sum_(i <- r | P i) f (E i).
Lemma rmorphMsign n : {morph f : x / (- 1) ^+ n × x}.
Lemma rmorphismMP : multiplicative f.
Lemma rmorph1 : f 1 = 1.
Lemma rmorphM : {morph f: x y / x × y}.
Lemma rmorph_prod I r (P : pred I) E :
f (\prod_(i <- r | P i) E i) = \prod_(i <- r | P i) f (E i).
Lemma rmorphX n : {morph f: x / x ^+ n}.
Lemma rmorph_nat n : f n%:R = n%:R.
Lemma rmorphN1 : f (- 1) = (- 1).
Lemma rmorph_sign n : f ((- 1) ^+ n) = (- 1) ^+ n.
Lemma rmorph_char p : p \in [char R] → p \in [char S].
Lemma rmorph_eq_nat x n : injective f → (f x == n%:R) = (x == n%:R).
Lemma rmorph_eq1 x : injective f → (f x == 1) = (x == 1).
Lemma can2_rmorphism f' : cancel f f' → cancel f' f → multiplicative f'.
End Properties.
Section Projections.
Variables (R S T : ringType) (f : {rmorphism S → T}) (g : {rmorphism R → S}).
Fact idfun_is_multiplicative : multiplicative (@idfun R).
#[export]
HB.instance Definition _ := isMultiplicative.Build R R idfun
idfun_is_multiplicative.
Fact comp_is_multiplicative : multiplicative (f \o g).
#[export]
HB.instance Definition _ := isMultiplicative.Build R T (f \o g)
comp_is_multiplicative.
End Projections.
Section InAlgebra.
Variables (R : ringType) (A : lalgType R).
Fact in_alg_is_additive : additive (in_alg_loc A).
#[export]
HB.instance Definition _ := isAdditive.Build R A (in_alg_loc A)
in_alg_is_additive.
Fact in_alg_is_rmorphism : multiplicative (in_alg_loc A).
#[export]
HB.instance Definition _ := isMultiplicative.Build R A (in_alg_loc A)
in_alg_is_rmorphism.
Lemma in_algE a : in_alg_loc A a = a%:A.
End InAlgebra.
End RmorphismTheory.
Module Scale.
#[export]
HB.structure Definition Law R V := {op of isLaw R V op}.
Definition law := Law.type.
Section ScaleLaw.
Variables (R : ringType) (V : zmodType) (s_law : law R V).
Lemma N1op : s_op (-1) =1 -%R.
Fact opB a : additive (s_op a).
Variables (aR : ringType) (nu : {rmorphism aR → R}).
Fact compN1op : (nu \; s_op) (-1) =1 -%R.
End ScaleLaw.
Module Exports. End Exports.
End Scale.
Export Scale.Exports.
#[export]
HB.instance Definition _ (R : ringType) := Scale.isLaw.Build R R *%R
(@mulN1r R) (@mulrBr R).
#[export]
HB.instance Definition _ (R : ringType) (U : lmodType R) :=
Scale.isLaw.Build R U *:%R (@scaleN1r R U) (@scalerBr R U).
#[export]
HB.instance Definition _ (R : ringType) (V : zmodType) (s : Scale.law R V)
(aR : ringType) (nu : {rmorphism aR → R}) :=
Scale.isLaw.Build aR V (nu \; s)
(@Scale.compN1op _ _ s _ nu) (fun a ⇒ Scale.opB _ _).
#[export, non_forgetful_inheritance]
HB.instance Definition _ (R : ringType) (V : zmodType) (s : Scale.law R V) a :=
isAdditive.Build V V (s a) (Scale.opB s a).
Definition scalable_for (R : ringType) (U : lmodType R) (V : zmodType)
(s : R → V → V) (f : U → V) :=
∀ a, {morph f : u / a *: u >-> s a u}.
Definition linear_for (R : ringType) (U : lmodType R) (V : zmodType)
(s : R → V → V) (f : U → V) :=
∀ a, {morph f : u v / a *: u + v >-> s a u + v}.
Lemma additive_linear (R : ringType) (U : lmodType R) V
(s : Scale.law R V) (f : U → V) : linear_for s f → additive f.
Lemma scalable_linear (R : ringType) (U : lmodType R) V
(s : Scale.law R V) (f : U → V) : linear_for s f → scalable_for s f.
Module LinearExports.
Notation scalable f := (scalable_for *:%R f).
Notation linear f := (linear_for *:%R f).
Notation scalar f := (linear_for *%R f).
Module Linear.
Section Linear.
Variables (R : ringType) (U : lmodType R) (V : zmodType) (s : R → V → V).
Definition map (phUV : phant (U → V)) := Linear.type U s.
Definition apply (phUV : phant (U → V)) := @Linear.sort R U V s.
Support for right-to-left rewriting with the generic linearZ rule.
Definition map_class := mapUV.
Definition map_at (a : R) := mapUV.
Structure map_for a s_a := MapFor {map_for_map : mapUV; _ : s a = s_a}.
Definition unify_map_at a (f : map_at a) := MapFor f (erefl (s a)).
Structure wrapped := Wrap {unwrap : mapUV}.
Definition wrap (f : map_class) := Wrap f.
End Linear.
End Linear.
Notation "{ 'linear' fUV | s }" := (Linear.map s (Phant fUV))
(at level 0, format "{ 'linear' fUV | s }") : type_scope.
Notation "{ 'linear' fUV }" := {linear fUV | *:%R}
(at level 0, format "{ 'linear' fUV }") : type_scope.
Notation "{ 'scalar' U }" := {linear U → _ | *%R}
(at level 0, format "{ 'scalar' U }") : type_scope.
Notation "[ 'linear' 'of' f 'as' g ]" := (Linear.clone _ _ _ _ f%function g)
(at level 0, format "[ 'linear' 'of' f 'as' g ]") : form_scope.
Notation "[ 'linear' 'of' f ]" := (Linear.clone _ _ _ _ f%function _)
(at level 0, format "[ 'linear' 'of' f ]") : form_scope.
Definition map_at (a : R) := mapUV.
Structure map_for a s_a := MapFor {map_for_map : mapUV; _ : s a = s_a}.
Definition unify_map_at a (f : map_at a) := MapFor f (erefl (s a)).
Structure wrapped := Wrap {unwrap : mapUV}.
Definition wrap (f : map_class) := Wrap f.
End Linear.
End Linear.
Notation "{ 'linear' fUV | s }" := (Linear.map s (Phant fUV))
(at level 0, format "{ 'linear' fUV | s }") : type_scope.
Notation "{ 'linear' fUV }" := {linear fUV | *:%R}
(at level 0, format "{ 'linear' fUV }") : type_scope.
Notation "{ 'scalar' U }" := {linear U → _ | *%R}
(at level 0, format "{ 'scalar' U }") : type_scope.
Notation "[ 'linear' 'of' f 'as' g ]" := (Linear.clone _ _ _ _ f%function g)
(at level 0, format "[ 'linear' 'of' f 'as' g ]") : form_scope.
Notation "[ 'linear' 'of' f ]" := (Linear.clone _ _ _ _ f%function _)
(at level 0, format "[ 'linear' 'of' f ]") : form_scope.
Support for right-to-left rewriting with the generic linearZ rule.
Coercion Linear.map_for_map : Linear.map_for >-> Linear.type.
Coercion Linear.unify_map_at : Linear.map_at >-> Linear.map_for.
Canonical Linear.unify_map_at.
Coercion Linear.unwrap : Linear.wrapped >-> Linear.type.
Coercion Linear.wrap : Linear.map_class >-> Linear.wrapped.
Canonical Linear.wrap.
End LinearExports.
Section LinearTheory.
Variable R : ringType.
Section GenericProperties.
Variables (U : lmodType R) (V : zmodType) (s : R → V → V) (k : unit).
Variable f : {linear U → V | s}.
Lemma linear0 : f 0 = 0.
Lemma linearN : {morph f : x / - x}.
Lemma linearD : {morph f : x y / x + y}.
Lemma linearB : {morph f : x y / x - y}.
Lemma linearMn n : {morph f : x / x *+ n}.
Lemma linearMNn n : {morph f : x / x *- n}.
Lemma linear_sum I r (P : pred I) E :
f (\sum_(i <- r | P i) E i) = \sum_(i <- r | P i) f (E i).
Lemma linearZ_LR : scalable_for s f.
Lemma linearP a : {morph f : u v / a *: u + v >-> s a u + v}.
End GenericProperties.
Section BidirectionalLinearZ.
Variables (U : lmodType R) (V : zmodType) (s : R → V → V).
Coercion Linear.unify_map_at : Linear.map_at >-> Linear.map_for.
Canonical Linear.unify_map_at.
Coercion Linear.unwrap : Linear.wrapped >-> Linear.type.
Coercion Linear.wrap : Linear.map_class >-> Linear.wrapped.
Canonical Linear.wrap.
End LinearExports.
Section LinearTheory.
Variable R : ringType.
Section GenericProperties.
Variables (U : lmodType R) (V : zmodType) (s : R → V → V) (k : unit).
Variable f : {linear U → V | s}.
Lemma linear0 : f 0 = 0.
Lemma linearN : {morph f : x / - x}.
Lemma linearD : {morph f : x y / x + y}.
Lemma linearB : {morph f : x y / x - y}.
Lemma linearMn n : {morph f : x / x *+ n}.
Lemma linearMNn n : {morph f : x / x *- n}.
Lemma linear_sum I r (P : pred I) E :
f (\sum_(i <- r | P i) E i) = \sum_(i <- r | P i) f (E i).
Lemma linearZ_LR : scalable_for s f.
Lemma linearP a : {morph f : u v / a *: u + v >-> s a u + v}.
End GenericProperties.
Section BidirectionalLinearZ.
Variables (U : lmodType R) (V : zmodType) (s : R → V → V).
The general form of the linearZ lemma uses some bespoke interfaces to
allow right-to-left rewriting when a composite scaling operation such as
conjC \; *%R has been expanded, say in a^* * f u. This redex is matched
by using the Scale.law interface to recognize a "head" scaling operation
h (here *%R), stow away its "scalar" c, then reconcile h c and s a, once
s is known, that is, once the Linear.map structure for f has been found.
In general, s and a need not be equal to h and c; indeed they need not
have the same type! The unification is performed by the unify_map_at
default instance for the Linear.map_for U s a h_c sub-interface of
Linear.map; the h_c pattern uses the Scale.law structure to insure it is
inferred when rewriting right-to-left.
The wrap on the rhs allows rewriting f (a *: b *: u) into a *: b *: f u
with rewrite !linearZ /= instead of rewrite linearZ /= linearZ /=.
Without it, the first rewrite linearZ would produce
(a *: apply (map_for_map (@check_map_at .. a f)) (b *: u)%R)%Rlin
and matching the second rewrite LHS would bypass the unify_map_at default
instance for b, reuse the one for a, and subsequently fail to match the
b *: u argument. The extra wrap / unwrap ensures that this can't happen.
In the RL direction, the wrap / unwrap will be inserted on the redex side
as needed, without causing unnecessary delta-expansion: using an explicit
identity function would have Coq normalize the redex to head normal, then
reduce the identity to expose the map_for_map projection, and the
expanded Linear.map structure would then be exposed in the result.
Most of this machinery will be invisible to a casual user, because all
the projections and default instances involved are declared as coercions.
Variables (S : ringType) (h : Scale.law S V).
Lemma linearZ c a (h_c := h c) (f : Linear.map_for U s a h_c) u :
f (a *: u) = h_c (Linear.wrap f u).
End BidirectionalLinearZ.
Section LmodProperties.
Variables (U V : lmodType R) (f : {linear U → V}).
Lemma linearZZ : scalable f.
Lemma linearPZ : linear f.
Lemma can2_scalable f' : cancel f f' → cancel f' f → scalable f'.
Lemma can2_linear f' : cancel f f' → cancel f' f → linear f'.
End LmodProperties.
Section ScalarProperties.
Variable (U : lmodType R) (f : {scalar U}).
Lemma scalarZ : scalable_for *%R f.
Lemma scalarP : scalar f.
End ScalarProperties.
Section LinearLmod.
Variables (W U : lmodType R) (V : zmodType).
Section Plain.
Variable (s : R → V → V).
Variables (f : {linear U → V | s}) (h : {linear W → U}).
Lemma idfun_is_scalable : scalable (@idfun U).
#[export]
HB.instance Definition _ := isLinear.Build R U U *:%R idfun idfun_is_scalable.
Lemma opp_is_scalable : scalable (-%R : U → U).
#[export]
HB.instance Definition _ := isLinear.Build R U U *:%R -%R opp_is_scalable.
Lemma comp_is_scalable : scalable_for s (f \o h).
#[export]
HB.instance Definition _ := isLinear.Build R W V s (f \o h) comp_is_scalable.
End Plain.
Section Scale.
Variable (s : Scale.law R V).
Variables (f : {linear U → V | s}) (g : {linear U → V | s}).
Lemma null_fun_is_scalable : scalable_for s (\0 : U → V).
#[export]
HB.instance Definition _ := isLinear.Build R U V s \0 null_fun_is_scalable.
Lemma add_fun_is_scalable : scalable_for s (f \+ g).
#[export]
HB.instance Definition _ := isLinear.Build R U V s (f \+ g) add_fun_is_scalable.
Lemma sub_fun_is_scalable : scalable_for s (f \- g).
#[export]
HB.instance Definition _ := isLinear.Build R U V s (f \- g) sub_fun_is_scalable.
Lemma opp_fun_is_scalable : scalable_for s (\- g).
#[export]
HB.instance Definition _ := isLinear.Build R U V s (\- g) opp_fun_is_scalable.
End Scale.
End LinearLmod.
Section LinearLalg.
Variables (A : lalgType R) (U : lmodType R).
Variables (a : A) (f : {linear U → A}).
Fact mulr_fun_is_scalable : scalable (a \o× f).
#[export]
HB.instance Definition _ := isLinear.Build R U A *:%R (a \o× f)
mulr_fun_is_scalable.
End LinearLalg.
End LinearTheory.
FIXME: strange implicit arguments for RMorphism (just like Additive)
Module LRMorphismExports.
Module LRMorphism.
Definition map (R : ringType) (A : lalgType R) (B : ringType) (s : R → B → B)
(phAB : phant (A → B)) := LRMorphism.type A s.
Definition apply (R : ringType) (A : lalgType R) (B : ringType) (s : R → B → B)
(phAB : phant (A → B)) := @LRMorphism.sort R A B s.
End LRMorphism.
Notation "{ 'lrmorphism' fAB | s }" := (LRMorphism.map s (Phant fAB%type))
(at level 0, format "{ 'lrmorphism' fAB | s }") : type_scope.
Notation "{ 'lrmorphism' fAB }" := {lrmorphism fAB%type | *:%R}
(at level 0, format "{ 'lrmorphism' fAB }") : type_scope.
Notation "[ 'lrmorphism' 'of' f ]" := (LRMorphism.clone _ _ _ _ f%function _)
(at level 0, format "[ 'lrmorphism' 'of' f ]") : form_scope.
End LRMorphismExports.
Section LRMorphismTheory.
Variables (R : ringType) (A B : lalgType R) (C : ringType) (s : R → C → C).
Variables (k : unit) (f : {lrmorphism A → B}) (g : {lrmorphism B → C | s}).
#[export] HB.instance Definition _ := RMorphism.on (@idfun A).
#[export] HB.instance Definition _ := RMorphism.on (g \o f).
Lemma rmorph_alg a : f a%:A = a%:A.
End LRMorphismTheory.
#[short(type="comRingType")]
HB.structure Definition ComRing := {R of Ring R & Ring_hasCommutativeMul R}.
Definition mulr1 := Monoid.mulC_id mulrC mul1r.
Definition mulrDr := Monoid.mulC_dist mulrC mulrDl.
Module ComRingExports.
Bind Scope ring_scope with ComRing.sort.
Notation "[ 'comRingType' 'of' T 'for' cT ]" := (ComRing.clone T%type cT)
(at level 0, format "[ 'comRingType' 'of' T 'for' cT ]") : form_scope.
Notation "[ 'comRingType' 'of' T ]" := (ComRing.clone T%type _)
(at level 0, format "[ 'comRingType' 'of' T ]") : form_scope.
End ComRingExports.
Section ComRingTheory.
Variable R : comRingType.
Implicit Types x y : R.
#[export]
HB.instance Definition _ := SemiGroup.isCommutativeLaw.Build R *%R mulrC.
Lemma mulrCA : @left_commutative R R *%R.
Lemma mulrAC : @right_commutative R R *%R.
Lemma mulrACA : @interchange R *%R *%R.
Lemma exprMn n : {morph (fun x ⇒ x ^+ n) : x y / x × y}.
Lemma prodrXl n I r (P : pred I) (F : I → R) :
\prod_(i <- r | P i) F i ^+ n = (\prod_(i <- r | P i) F i) ^+ n.
Lemma prodr_undup_exp_count (I : eqType) r (P : pred I) (F : I → R) :
\prod_(i <- undup r | P i) F i ^+ count_mem i r = \prod_(i <- r | P i) F i.
Lemma exprDn x y n :
(x + y) ^+ n = \sum_(i < n.+1) (x ^+ (n - i) × y ^+ i) *+ 'C(n, i).
Lemma exprBn x y n :
(x - y) ^+ n =
\sum_(i < n.+1) ((-1) ^+ i × x ^+ (n - i) × y ^+ i) *+ 'C(n, i).
Lemma subrXX x y n :
x ^+ n - y ^+ n = (x - y) × (\sum_(i < n) x ^+ (n.-1 - i) × y ^+ i).
Lemma sqrrD x y : (x + y) ^+ 2 = x ^+ 2 + x × y *+ 2 + y ^+ 2.
Lemma sqrrB x y : (x - y) ^+ 2 = x ^+ 2 - x × y *+ 2 + y ^+ 2.
Lemma subr_sqr x y : x ^+ 2 - y ^+ 2 = (x - y) × (x + y).
Lemma subr_sqrDB x y : (x + y) ^+ 2 - (x - y) ^+ 2 = x × y *+ 4.
Section FrobeniusAutomorphism.
Variables (p : nat) (charRp : p \in [char R]).
Lemma Frobenius_aut_is_additive : additive (Frobenius_aut charRp).
Lemma Frobenius_aut_is_multiplicative : multiplicative (Frobenius_aut charRp).
#[export]
HB.instance Definition _ := isAdditive.Build R R (Frobenius_aut charRp)
Frobenius_aut_is_additive.
#[export]
HB.instance Definition _ := isMultiplicative.Build R R (Frobenius_aut charRp)
Frobenius_aut_is_multiplicative.
End FrobeniusAutomorphism.
Lemma exprDn_char x y n : [char R].-nat n → (x + y) ^+ n = x ^+ n + y ^+ n.
Lemma rmorph_comm (S : ringType) (f : {rmorphism R → S}) x y :
comm (f x) (f y).
Section ScaleLinear.
Variables (U V : lmodType R) (b : R) (f : {linear U → V}).
Lemma scale_is_scalable : scalable ( *:%R b : V → V).
#[export]
HB.instance Definition _ := isLinear.Build R V V *:%R ( *:%R b)
scale_is_scalable.
Lemma scale_fun_is_scalable : scalable (b \*: f).
#[export]
HB.instance Definition _ := isLinear.Build R U V *:%R (b \*: f)
scale_fun_is_scalable.
End ScaleLinear.
End ComRingTheory.
#[infer(R), short(type="algType")]
HB.structure Definition Algebra (R : ringType) :=
{A of Lalgebra_isAlgebra R A & Lalgebra R A}.
Module AlgExports.
Bind Scope ring_scope with Algebra.sort.
Notation "[ 'algType' R 'of' T 'for' cT ]" :=
(Algebra.clone [the ringType of R] T%type cT)
(at level 0, format "[ 'algType' R 'of' T 'for' cT ]")
: form_scope.
Notation "[ 'algType' R 'of' T ]" := [algType R of T%type for _]
(at level 0, format "[ 'algType' R 'of' T ]") : form_scope.
End AlgExports.
FIXME: bad naming
Lemma scalarAr k (x y : V) : k *: (x × y) = x × (k *: y).
#[infer(R), short(type="comAlgType")]
HB.structure Definition ComAlgebra R :=
{V of is_ComAlgebra R V & ComRing V & Lalgebra R V}.
Module ComAlgExports.
Bind Scope ring_scope with ComAlgebra.sort.
Notation "[ 'comAlgType' R 'of' T ]" :=
(ComAlgebra.clone [the ringType of R] T%type _)
(at level 0, format "[ 'comAlgType' R 'of' T ]") : form_scope.
End ComAlgExports.
Section AlgebraTheory.
Variables (R : comRingType) (A : algType R).
#[export]
HB.instance Definition converse_ : Ring_hasCommutativeMul R^c :=
Ring_hasCommutativeMul.Build R^c (fun _ _ ⇒ mulrC _ _).
#[export]
HB.instance Definition regular_comRingType : Ring_hasCommutativeMul R^o :=
Ring_hasCommutativeMul.Build R^o mulrC.
#[export]
HB.instance Definition regular_comAlgType : is_ComAlgebra R R^o :=
is_ComAlgebra.Build R R^o.
End AlgebraTheory.
Section AlgebraTheory.
Variables (R : comRingType) (A : algType R).
Implicit Types (k : R) (x y : A).
Lemma scalerCA k x y : k *: x × y = x × (k *: y).
Lemma mulr_algr a x : x × a%:A = a *: x.
Lemma comm_alg a x : comm a%:A x.
Lemma exprZn k x n : (k *: x) ^+ n = k ^+ n *: x ^+ n.
Lemma scaler_prod I r (P : pred I) (F : I → R) (G : I → A) :
\prod_(i <- r | P i) (F i *: G i) =
\prod_(i <- r | P i) F i *: \prod_(i <- r | P i) G i.
Lemma scaler_prodl (I : finType) (S : pred I) (F : I → A) k :
\prod_(i in S) (k *: F i) = k ^+ #|S| *: \prod_(i in S) F i.
Lemma scaler_prodr (I : finType) (S : pred I) (F : I → R) x :
\prod_(i in S) (F i *: x) = \prod_(i in S) F i *: x ^+ #|S|.
Variables (U : lmodType R) (a : A) (f : {linear U → A}).
Lemma mull_fun_is_scalable : scalable (a \*o f).
#[export]
HB.instance Definition _ := isLinear.Build R U A *:%R (a \*o f)
mull_fun_is_scalable.
End AlgebraTheory.
#[short(type="unitRingType")]
HB.structure Definition UnitRing := {R of Ring_hasMulInverse R & Ring R}.
Module UnitRingExports.
Bind Scope ring_scope with UnitRing.sort.
Notation "[ 'unitRingType' 'of' T 'for' cT ]" := (UnitRing.clone T%type cT)
(at level 0, format "[ 'unitRingType' 'of' T 'for' cT ]") : form_scope.
Notation "[ 'unitRingType' 'of' T ]" := (UnitRing.clone T%type _)
(at level 0, format "[ 'unitRingType' 'of' T ]") : form_scope.
End UnitRingExports.
Definition unit_pred {R : unitRingType} :=
Eval cbv [ unit_subdef Ring_hasMulInverse.unit_subdef ] in
(fun u : R ⇒ unit_subdef u).
Arguments unit_pred _ _ /.
Definition unit {R : unitRingType} := [qualify a u : R | unit_pred u].
Section UnitRingTheory.
Variable R : unitRingType.
Implicit Types x y : R.
Lemma divrr : {in unit, right_inverse 1 (@inv R) *%R}.
Definition mulrV := divrr.
Lemma mulVr : {in unit, left_inverse 1 (@inv R) *%R}.
Lemma invr_out x : x \isn't a unit → x^-1 = x.
Lemma unitrP x : reflect (∃ y, y × x = 1 ∧ x × y = 1) (x \is a unit).
Lemma mulKr : {in unit, left_loop (@inv R) *%R}.
Lemma mulVKr : {in unit, rev_left_loop (@inv R) *%R}.
Lemma mulrK : {in unit, right_loop (@inv R) *%R}.
Lemma mulrVK : {in unit, rev_right_loop (@inv R) *%R}.
Definition divrK := mulrVK.
Lemma mulrI : {in @unit R, right_injective *%R}.
Lemma mulIr : {in @unit R, left_injective *%R}.
Due to noncommutativity, fractions are inverted.
Lemma telescope_prodr n m (f : nat → R) :
(∀ k, n < k < m → f k \is a unit) → n < m →
\prod_(n ≤ k < m) (f k / f k.+1) = f n / f m.
Lemma commrV x y : comm x y → comm x y^-1.
Lemma unitrE x : (x \is a unit) = (x / x == 1).
Lemma invrK : involutive (@inv R).
Lemma invr_inj : injective (@inv R).
Lemma unitrV x : (x^-1 \in unit) = (x \in unit).
Lemma unitr1 : 1 \in @unit R.
Lemma invr1 : 1^-1 = 1 :> R.
Lemma div1r x : 1 / x = x^-1.
Lemma divr1 x : x / 1 = x.
Lemma natr_div m d :
d %| m → d%:R \is a @unit R → (m %/ d)%:R = m%:R / d%:R :> R.
Lemma divrI : {in unit, right_injective (fun x y ⇒ x / y)}.
Lemma divIr : {in unit, left_injective (fun x y ⇒ x / y)}.
Lemma unitr0 : (0 \is a @unit R) = false.
Lemma invr0 : 0^-1 = 0 :> R.
Lemma unitrN1 : -1 \is a @unit R.
Lemma invrN1 : (-1)^-1 = -1 :> R.
Lemma invr_sign n : ((-1) ^- n) = (-1) ^+ n :> R.
Lemma unitrMl x y : y \is a unit → (x × y \is a unit) = (x \is a unit).
Lemma unitrMr x y : x \is a unit → (x × y \is a unit) = (y \is a unit).
Lemma invrM : {in unit &, ∀ x y, (x × y)^-1 = y^-1 × x^-1}.
Lemma unitrM_comm x y :
comm x y → (x × y \is a unit) = (x \is a unit) && (y \is a unit).
Lemma unitrX x n : x \is a unit → x ^+ n \is a unit.
Lemma unitrX_pos x n : n > 0 → (x ^+ n \in unit) = (x \in unit).
Lemma exprVn x n : x^-1 ^+ n = x ^- n.
Lemma exprB m n x : n ≤ m → x \is a unit → x ^+ (m - n) = x ^+ m / x ^+ n.
Lemma invr_neq0 x : x != 0 → x^-1 != 0.
Lemma invr_eq0 x : (x^-1 == 0) = (x == 0).
Lemma invr_eq1 x : (x^-1 == 1) = (x == 1).
Lemma rev_unitrP (x y : R^c) : y × x = 1 ∧ x × y = 1 → x \is a unit.
End UnitRingTheory.
Arguments invrK {R}.
Arguments invr_inj {R} [x1 x2].
Module RegularConverseUnitRingExports.
Section UnitRingTheory.
Variable R : unitRingType.
Implicit Types x y : R.
End UnitRingTheory.
End RegularConverseUnitRingExports.
Section UnitRingClosedPredicates.
Variable R : unitRingType.
Implicit Types x y : R.
Variables S : {pred R}.
Definition invr_closed := {in S, ∀ x, x^-1 \in S}.
Definition divr_2closed := {in S &, ∀ x y, x / y \in S}.
Definition divr_closed := 1 \in S ∧ divr_2closed.
Definition sdivr_closed := -1 \in S ∧ divr_2closed.
Definition divring_closed := [/\ 1 \in S, subr_2closed S & divr_2closed].
Lemma divr_closedV : divr_closed → invr_closed.
Lemma divr_closedM : divr_closed → mulr_closed S.
Lemma sdivr_closed_div : sdivr_closed → divr_closed.
Lemma sdivr_closedM : sdivr_closed → smulr_closed S.
Lemma divring_closedBM : divring_closed → subring_closed S.
Lemma divring_closed_div : divring_closed → sdivr_closed.
End UnitRingClosedPredicates.
Section UnitRingMorphism.
Variables (R S : unitRingType) (f : {rmorphism R → S}).
Lemma rmorph_unit x : x \in unit → f x \in unit.
Lemma rmorphV : {in unit, {morph f: x / x^-1}}.
Lemma rmorph_div x y : y \in unit → f (x / y) = f x / f y.
End UnitRingMorphism.
#[short(type="comUnitRingType")]
HB.structure Definition ComUnitRing := {R of ComRing R & UnitRing R}.
Module ComUnitRingExports.
Bind Scope ring_scope with ComUnitRing.sort.
Notation "[ 'comUnitRingType' 'of' T ]" := (ComUnitRing.clone T%type _)
(at level 0, format "[ 'comUnitRingType' 'of' T ]") : form_scope.
End ComUnitRingExports.
Fact mulC_mulrV :
(∀ k, n < k < m → f k \is a unit) → n < m →
\prod_(n ≤ k < m) (f k / f k.+1) = f n / f m.
Lemma commrV x y : comm x y → comm x y^-1.
Lemma unitrE x : (x \is a unit) = (x / x == 1).
Lemma invrK : involutive (@inv R).
Lemma invr_inj : injective (@inv R).
Lemma unitrV x : (x^-1 \in unit) = (x \in unit).
Lemma unitr1 : 1 \in @unit R.
Lemma invr1 : 1^-1 = 1 :> R.
Lemma div1r x : 1 / x = x^-1.
Lemma divr1 x : x / 1 = x.
Lemma natr_div m d :
d %| m → d%:R \is a @unit R → (m %/ d)%:R = m%:R / d%:R :> R.
Lemma divrI : {in unit, right_injective (fun x y ⇒ x / y)}.
Lemma divIr : {in unit, left_injective (fun x y ⇒ x / y)}.
Lemma unitr0 : (0 \is a @unit R) = false.
Lemma invr0 : 0^-1 = 0 :> R.
Lemma unitrN1 : -1 \is a @unit R.
Lemma invrN1 : (-1)^-1 = -1 :> R.
Lemma invr_sign n : ((-1) ^- n) = (-1) ^+ n :> R.
Lemma unitrMl x y : y \is a unit → (x × y \is a unit) = (x \is a unit).
Lemma unitrMr x y : x \is a unit → (x × y \is a unit) = (y \is a unit).
Lemma invrM : {in unit &, ∀ x y, (x × y)^-1 = y^-1 × x^-1}.
Lemma unitrM_comm x y :
comm x y → (x × y \is a unit) = (x \is a unit) && (y \is a unit).
Lemma unitrX x n : x \is a unit → x ^+ n \is a unit.
Lemma unitrX_pos x n : n > 0 → (x ^+ n \in unit) = (x \in unit).
Lemma exprVn x n : x^-1 ^+ n = x ^- n.
Lemma exprB m n x : n ≤ m → x \is a unit → x ^+ (m - n) = x ^+ m / x ^+ n.
Lemma invr_neq0 x : x != 0 → x^-1 != 0.
Lemma invr_eq0 x : (x^-1 == 0) = (x == 0).
Lemma invr_eq1 x : (x^-1 == 1) = (x == 1).
Lemma rev_unitrP (x y : R^c) : y × x = 1 ∧ x × y = 1 → x \is a unit.
End UnitRingTheory.
Arguments invrK {R}.
Arguments invr_inj {R} [x1 x2].
Module RegularConverseUnitRingExports.
Section UnitRingTheory.
Variable R : unitRingType.
Implicit Types x y : R.
End UnitRingTheory.
End RegularConverseUnitRingExports.
Section UnitRingClosedPredicates.
Variable R : unitRingType.
Implicit Types x y : R.
Variables S : {pred R}.
Definition invr_closed := {in S, ∀ x, x^-1 \in S}.
Definition divr_2closed := {in S &, ∀ x y, x / y \in S}.
Definition divr_closed := 1 \in S ∧ divr_2closed.
Definition sdivr_closed := -1 \in S ∧ divr_2closed.
Definition divring_closed := [/\ 1 \in S, subr_2closed S & divr_2closed].
Lemma divr_closedV : divr_closed → invr_closed.
Lemma divr_closedM : divr_closed → mulr_closed S.
Lemma sdivr_closed_div : sdivr_closed → divr_closed.
Lemma sdivr_closedM : sdivr_closed → smulr_closed S.
Lemma divring_closedBM : divring_closed → subring_closed S.
Lemma divring_closed_div : divring_closed → sdivr_closed.
End UnitRingClosedPredicates.
Section UnitRingMorphism.
Variables (R S : unitRingType) (f : {rmorphism R → S}).
Lemma rmorph_unit x : x \in unit → f x \in unit.
Lemma rmorphV : {in unit, {morph f: x / x^-1}}.
Lemma rmorph_div x y : y \in unit → f (x / y) = f x / f y.
End UnitRingMorphism.
#[short(type="comUnitRingType")]
HB.structure Definition ComUnitRing := {R of ComRing R & UnitRing R}.
Module ComUnitRingExports.
Bind Scope ring_scope with ComUnitRing.sort.
Notation "[ 'comUnitRingType' 'of' T ]" := (ComUnitRing.clone T%type _)
(at level 0, format "[ 'comUnitRingType' 'of' T ]") : form_scope.
End ComUnitRingExports.
Fact mulC_mulrV :