aboutsummaryrefslogtreecommitdiff
path: root/src/Util/AdditionChainExponentiation.v
Commit message (Collapse)AuthorAge
* Add a Require Import FunInd (Function isn't loaded by default anymore)Gravatar Pierre Letouzey2017-10-18
| | | | See PR #220 https://github.com/coq/coq/pull/220
* ScalarMult: Z -> G -> G (closes #193)Gravatar Andres Erbsen2017-06-14
|
* Don't rely on autogenerated namesGravatar Jason Gross2017-06-05
| | | | | | This fixes all of the private-names warnings emitted by compiling fiat-crypto with https://github.com/coq/coq/pull/268 (minus the ones in coqprime, which I didn't touch).
* rename-everythingGravatar Andres Erbsen2017-04-06
|
* do not use VerdiTactics in files we plan to keepGravatar Andres Erbsen2017-04-06
|
* Add [Proof using] to most proofsGravatar Jason Gross2017-04-04
| | | | | | | | This closes #146 and makes `make quick` faster. The changes were generated by adding [Global Set Suggest Proof Using.] to GlobalSettings.v, and then following [the instructions for a script I wrote](https://github.com/JasonGross/coq-tools#proof-using-helper).
* split the algebra library; use fsatz moreGravatar Andres Erbsen2017-03-02
|
* Fully qualify [Require]sGravatar Jason Gross2016-09-08
| | | | This way they won't become ambiguous if we add new files
* Removed lingering SearchAbout.Gravatar jadep2016-08-31
|
* Updated AdditionChainExponentiation.v such that the exponentiation ↵Gravatar jadep2016-08-23
| | | | correctness is in terms of N rather than nat; this allows us to compute the correctness proof for large exponents.
* Refactor ModularArithmetic into Zmod, expand DecidableGravatar Andres Erbsen2016-08-04
| | | | | | | | | | | | ModularArithmetic now uses Algebra lemmas in various places instead of custom manual proofs. Similarly, Util.Decidable is used to state and prove the relevant decidability results. Backwards-incompatible changes: F_some_lemma -> Zmod.some_lemma Arguments ZToField _%Z _%Z : clear implicits. inv_spec says inv x * x = 1, not x * inv x = 1
* added proofs about addition chain exponentiation for later use in ↵Gravatar jadep2016-07-10
ModularBaseSystem [pow], which we need for sqrt and inversion.