aboutsummaryrefslogtreecommitdiff
path: root/src/Util/WordUtil.v
Commit message (Collapse)AuthorAge
* Remove WordUtilGravatar Benjamin Barenblat2019-04-26
| | | | Remove Util/NUtil.v and Util/WordUtil.v. This code is no longer in use.
* Add Z.land, Z.lor bounds stuff to zutil, also split up ZUtilGravatar Jason Gross2018-08-23
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | The file src/Util/ZUtil.v no longer exports any lemmas, nor does it contain any lemmas. Instead, it pulls in all of the various ZUtil files so that `Search` will pick up the relevant lemma, and allow users to `Require Import` the relevant file. This allows more parallelization in the build. It also prevents needlessly rebuilding lots of files whenever we change anything anywhere in ZUtil. From this point forward, no file in the development should `Require` `Crypto.Util.ZUtil` itself. After | File Name | Before || Change | % Change ----------------------------------------------------------------------------------------------------------------------- 73m47.61s | Total | 73m49.49s || -0m01.87s | -0.04% ----------------------------------------------------------------------------------------------------------------------- 0m14.49s | Util/ZUtil/LandLorBounds | N/A || +0m14.49s | ∞ 0m00.42s | Util/ZUtil | 0m11.07s || -0m10.65s | -96.20% 0m03.54s | Util/ZUtil/LandLorShiftBounds | N/A || +0m03.54s | ∞ 0m03.49s | Util/ZUtil/Shift | N/A || +0m03.49s | ∞ 4m09.67s | Experiments/NewPipeline/RewriterRulesGood | 4m07.61s || +0m02.05s | +0.83% 1m22.68s | Experiments/NewPipeline/RewriterWf2 | 1m20.22s || +0m02.46s | +3.06% 1m21.09s | Compilers/Named/MapCastInterp | 1m23.14s || -0m02.04s | -2.46% 0m17.79s | Arithmetic/MontgomeryReduction/WordByWord/Abstract/Dependent/Proofs | 0m20.61s || -0m02.82s | -13.68% 0m08.00s | Arithmetic/MontgomeryReduction/Proofs | 0m10.90s || -0m02.90s | -26.60% 0m05.46s | LegacyArithmetic/Double/Proofs/SpreadLeftImmediate | 0m08.07s || -0m02.61s | -32.34% 8m39.34s | Experiments/SimplyTypedArithmetic | 8m38.00s || +0m01.34s | +0.25% 1m30.51s | Spec/Test/X25519 | 1m28.92s || +0m01.59s | +1.78% 1m16.98s | Experiments/NewPipeline/Rewriter | 1m18.02s || -0m01.03s | -1.33% 0m25.51s | Experiments/NewPipeline/UnderLetsProofs | 0m27.02s || -0m01.50s | -5.58% 0m10.75s | Arithmetic/MontgomeryReduction/WordByWord/Abstract/Proofs | 0m12.00s || -0m01.25s | -10.41% 0m09.28s | LegacyArithmetic/Double/Proofs/Multiply | 0m10.97s || -0m01.69s | -15.40% 0m05.70s | LegacyArithmetic/Double/Proofs/RippleCarryAddSub | 0m07.01s || -0m01.30s | -18.68% 0m03.36s | LegacyArithmetic/InterfaceProofs | 0m04.67s || -0m01.31s | -28.05% 0m01.43s | Util/ZUtil/Ones | N/A || +0m01.42s | ∞ 0m01.37s | Arithmetic/BarrettReduction/Wikipedia | 0m02.38s || -0m01.00s | -42.43% 6m02.75s | Experiments/NewPipeline/SlowPrimeSynthesisExamples | 6m03.58s || -0m00.82s | -0.22% 4m45.52s | Experiments/NewPipeline/Toplevel1 | 4m45.02s || +0m00.50s | +0.17% 3m46.16s | Curves/Montgomery/XZProofs | 3m45.20s || +0m00.96s | +0.42% 2m11.24s | Specific/X25519/C64/ladderstep | 2m11.78s || -0m00.53s | -0.40% 1m52.27s | Specific/NISTP256/AMD64/femul | 1m52.36s || -0m00.08s | -0.08% 1m43.21s | Experiments/NewPipeline/Toplevel2 | 1m43.70s || -0m00.48s | -0.47% 1m30.09s | Experiments/NewPipeline/Arithmetic | 1m29.59s || +0m00.50s | +0.55% 1m18.58s | Specific/X2448/Karatsuba/C64/femul | 1m19.45s || -0m00.87s | -1.09% 0m59.72s | Specific/X25519/C32/femul | 1m00.00s || -0m00.28s | -0.46% 0m52.94s | Demo | 0m52.24s || +0m00.69s | +1.33% 0m48.98s | Compilers/Z/Named/RewriteAddToAdcInterp | 0m49.12s || -0m00.14s | -0.28% 0m47.34s | Compilers/Z/ArithmeticSimplifierInterp | 0m47.24s || +0m00.10s | +0.21% 0m43.02s | Specific/X25519/C32/fesquare | 0m43.06s || -0m00.03s | -0.09% 0m42.02s | Arithmetic/Karatsuba | 0m42.08s || -0m00.05s | -0.14% 0m41.76s | Experiments/NewPipeline/AbstractInterpretationWf | 0m42.33s || -0m00.57s | -1.34% 0m38.51s | p521_32.c | 0m38.75s || -0m00.24s | -0.61% 0m37.14s | Experiments/NewPipeline/ExtractionOCaml/word_by_word_montgomery | 0m37.22s || -0m00.07s | -0.21% 0m36.10s | Spec/Ed25519 | 0m36.23s || -0m00.12s | -0.35% 0m35.83s | Experiments/NewPipeline/LanguageInversion | 0m35.71s || +0m00.11s | +0.33% 0m34.38s | Experiments/NewPipeline/ExtractionHaskell/word_by_word_montgomery | 0m34.91s || -0m00.52s | -1.51% 0m33.32s | Specific/X25519/C32/freeze | 0m33.32s || +0m00.00s | +0.00% 0m31.92s | p521_64.c | 0m32.20s || -0m00.28s | -0.86% 0m31.32s | Compilers/Z/ArithmeticSimplifierWf | 0m30.82s || +0m00.50s | +1.62% 0m28.96s | Compilers/CommonSubexpressionEliminationWf | 0m29.19s || -0m00.23s | -0.78% 0m27.73s | Specific/NISTP256/AMD128/femul | 0m27.70s || +0m00.03s | +0.10% 0m26.79s | Primitives/EdDSARepChange | 0m26.90s || -0m00.10s | -0.40% 0m25.27s | Specific/X25519/C32/fecarry | 0m25.34s || -0m00.07s | -0.27% 0m24.87s | Experiments/NewPipeline/AbstractInterpretationZRangeProofs | 0m25.26s || -0m00.39s | -1.54% 0m23.71s | p384_32.c | 0m23.60s || +0m00.10s | +0.46% 0m22.37s | Experiments/NewPipeline/LanguageWf | 0m22.49s || -0m00.11s | -0.53% 0m21.43s | Arithmetic/Core | 0m21.60s || -0m00.17s | -0.78% 0m21.41s | Specific/X25519/C32/fesub | 0m21.28s || +0m00.12s | +0.61% 0m20.86s | Experiments/NewPipeline/ExtractionHaskell/unsaturated_solinas | 0m20.26s || +0m00.59s | +2.96% 0m20.86s | Specific/NISTP256/AMD64/fesub | 0m21.69s || -0m00.83s | -3.82% 0m20.53s | Specific/X25519/C64/femul | 0m20.54s || -0m00.00s | -0.04% 0m19.67s | Specific/X25519/C32/Synthesis | 0m19.54s || +0m00.13s | +0.66% 0m19.44s | Curves/Edwards/XYZT/Basic | 0m19.05s || +0m00.39s | +2.04% 0m19.30s | Specific/NISTP256/AMD64/feadd | 0m19.35s || -0m00.05s | -0.25% 0m19.23s | Specific/X25519/C32/feadd | 0m19.20s || +0m00.03s | +0.15% 0m18.84s | Experiments/NewPipeline/ExtractionOCaml/unsaturated_solinas | 0m18.60s || +0m00.23s | +1.29% 0m18.07s | Compilers/Named/MapCastWf | 0m17.87s || +0m00.19s | +1.11% 0m18.01s | Compilers/Z/CNotations | 0m18.15s || -0m00.13s | -0.77% 0m17.50s | Specific/X25519/C64/freeze | 0m17.52s || -0m00.01s | -0.11% 0m17.03s | Specific/X25519/C64/fesquare | 0m17.14s || -0m00.10s | -0.64% 0m16.10s | Curves/Edwards/AffineProofs | 0m15.80s || +0m00.30s | +1.89% 0m15.71s | Specific/NISTP256/AMD64/feopp | 0m15.97s || -0m00.25s | -1.62% 0m15.62s | Compilers/Named/ContextProperties/SmartMap | 0m15.57s || +0m00.04s | +0.32% 0m15.35s | Compilers/Named/ContextProperties/NameUtil | 0m15.30s || +0m00.04s | +0.32% 0m15.04s | Specific/NISTP256/AMD128/fesub | 0m15.16s || -0m00.12s | -0.79% 0m14.88s | Specific/NISTP256/AMD128/feadd | 0m14.83s || +0m00.05s | +0.33% 0m14.20s | Specific/NISTP256/AMD64/fenz | 0m14.56s || -0m00.36s | -2.47% 0m14.16s | Specific/X25519/C64/fecarry | 0m14.13s || +0m00.02s | +0.21% 0m13.78s | Experiments/NewPipeline/ExtractionHaskell/saturated_solinas | 0m13.54s || +0m00.24s | +1.77% 0m13.69s | Arithmetic/Saturated/AddSub | 0m13.66s || +0m00.02s | +0.21% 0m13.67s | Specific/NISTP256/AMD128/fenz | 0m13.69s || -0m00.01s | -0.14% 0m13.16s | Experiments/NewPipeline/CStringification | 0m13.08s || +0m00.08s | +0.61% 0m13.10s | Specific/X25519/C64/fesub | 0m13.16s || -0m00.06s | -0.45% 0m12.34s | Experiments/NewPipeline/AbstractInterpretationProofs | 0m12.47s || -0m00.13s | -1.04% 0m12.29s | Specific/NISTP256/AMD128/feopp | 0m12.34s || -0m00.05s | -0.40% 0m12.26s | Compilers/Z/Syntax/Equality | 0m12.69s || -0m00.42s | -3.38% 0m11.94s | Specific/X25519/C64/feadd | 0m11.90s || +0m00.03s | +0.33% 0m11.87s | Primitives/MxDHRepChange | 0m11.76s || +0m00.10s | +0.93% 0m11.85s | Experiments/NewPipeline/GENERATEDIdentifiersWithoutTypesProofs | 0m11.66s || +0m00.18s | +1.62% 0m11.42s | Arithmetic/Saturated/MontgomeryAPI | 0m11.45s || -0m00.02s | -0.26% 0m10.69s | Experiments/NewPipeline/ExtractionOCaml/saturated_solinas | 0m10.30s || +0m00.38s | +3.78% 0m10.61s | Arithmetic/Saturated/Core | 0m10.66s || -0m00.05s | -0.46% 0m09.89s | Specific/X2448/Karatsuba/C64/Synthesis | 0m09.79s || +0m00.10s | +1.02% 0m09.35s | Util/ZRange/CornersMonotoneBounds | 0m09.90s || -0m00.55s | -5.55% 0m08.79s | Experiments/NewPipeline/ExtractionOCaml/word_by_word_montgomery.ml | 0m08.60s || +0m00.18s | +2.20% 0m08.64s | p384_64.c | 0m08.50s || +0m00.14s | +1.64% 0m08.63s | LegacyArithmetic/ArchitectureToZLikeProofs | 0m08.61s || +0m00.02s | +0.23% 0m08.49s | LegacyArithmetic/Double/Proofs/ShiftRightDoubleWordImmediate | 0m08.38s || +0m00.10s | +1.31% 0m08.19s | Compilers/Named/CompileInterpSideConditions | 0m07.78s || +0m00.40s | +5.26% 0m08.15s | Experiments/NewPipeline/GENERATEDIdentifiersWithoutTypes | 0m08.20s || -0m00.04s | -0.60% 0m07.98s | Compilers/Named/RegisterAssignInterp | 0m08.11s || -0m00.12s | -1.60% 0m07.81s | Arithmetic/BarrettReduction/RidiculousFish | 0m08.20s || -0m00.38s | -4.75% 0m07.45s | Compilers/InlineConstAndOpWf | 0m07.40s || +0m00.04s | +0.67% 0m07.01s | Specific/NISTP256/AMD64/Synthesis | 0m06.98s || +0m00.02s | +0.42% 0m06.55s | Compilers/Z/Bounds/InterpretationLemmas/PullCast | 0m06.44s || +0m00.10s | +1.70% 0m06.51s | Arithmetic/Saturated/MulSplit | 0m06.45s || +0m00.05s | +0.93% 0m06.40s | Util/FixedWordSizesEquality | 0m06.46s || -0m00.05s | -0.92% 0m06.28s | Arithmetic/BarrettReduction/Generalized | 0m06.64s || -0m00.35s | -5.42% 0m06.08s | Util/ZUtil/Modulo | 0m05.58s || +0m00.50s | +8.96% 0m06.07s | Compilers/InlineWf | 0m06.20s || -0m00.12s | -2.09% 0m06.04s | Util/ZUtil/Morphisms | 0m06.09s || -0m00.04s | -0.82% 0m05.94s | Specific/X25519/C64/Synthesis | 0m05.95s || -0m00.00s | -0.16% 0m05.66s | Compilers/LinearizeWf | 0m05.73s || -0m00.07s | -1.22% 0m05.64s | LegacyArithmetic/Pow2BaseProofs | 0m06.27s || -0m00.62s | -10.04% 0m05.60s | Experiments/NewPipeline/ExtractionHaskell/word_by_word_montgomery.hs | 0m05.45s || +0m00.14s | +2.75% 0m05.45s | Experiments/NewPipeline/ExtractionOCaml/unsaturated_solinas.ml | 0m05.54s || -0m00.08s | -1.62% 0m05.29s | Compilers/Z/HexNotationConstants | 0m05.44s || -0m00.15s | -2.75% 0m05.02s | Compilers/WfProofs | 0m04.98s || +0m00.03s | +0.80% 0m04.76s | Experiments/NewPipeline/RewriterWf1 | 0m04.74s || +0m00.01s | +0.42% 0m04.69s | Specific/Framework/ArithmeticSynthesis/Montgomery | 0m04.71s || -0m00.01s | -0.42% 0m04.63s | Arithmetic/BarrettReduction/HAC | 0m05.14s || -0m00.50s | -9.92% 0m04.48s | Compilers/Z/Bounds/Pipeline/Definition | 0m04.68s || -0m00.19s | -4.27% 0m04.34s | Compilers/Z/BinaryNotationConstants | 0m04.39s || -0m00.04s | -1.13% 0m04.14s | Compilers/Named/CompileWf | 0m04.19s || -0m00.05s | -1.19% 0m04.02s | Experiments/NewPipeline/MiscCompilerPassesProofs | 0m03.98s || +0m00.03s | +1.00% 0m03.99s | Experiments/NewPipeline/ExtractionHaskell/unsaturated_solinas.hs | 0m03.87s || +0m00.12s | +3.10% 0m03.90s | secp256k1_32.c | 0m03.91s || -0m00.01s | -0.25% 0m03.87s | Experiments/NewPipeline/ExtractionOCaml/saturated_solinas.ml | 0m03.98s || -0m00.10s | -2.76% 0m03.83s | Arithmetic/MontgomeryReduction/WordByWord/Proofs | 0m03.72s || +0m00.10s | +2.95% 0m03.76s | p256_32.c | 0m03.81s || -0m00.05s | -1.31% 0m03.67s | LegacyArithmetic/Double/Proofs/ShiftRight | 0m03.59s || +0m00.08s | +2.22% 0m03.58s | Compilers/Z/ArithmeticSimplifier | 0m03.60s || -0m00.02s | -0.55% 0m03.48s | Compilers/Z/Bounds/InterpretationLemmas/IsBoundedBy | 0m03.46s || +0m00.02s | +0.57% 0m03.41s | Experiments/NewPipeline/ExtractionHaskell/saturated_solinas.hs | 0m03.32s || +0m00.09s | +2.71% 0m03.28s | Specific/NISTP256/AMD128/Synthesis | 0m03.30s || -0m00.02s | -0.60% 0m03.24s | Util/ZUtil/Div | 0m02.78s || +0m00.46s | +16.54% 0m03.12s | LegacyArithmetic/Double/Proofs/ShiftLeft | 0m03.13s || -0m00.00s | -0.31% 0m03.05s | Compilers/InlineInterp | 0m02.91s || +0m00.13s | +4.81% 0m03.04s | LegacyArithmetic/Double/Proofs/Decode | 0m03.48s || -0m00.43s | -12.64% 0m02.98s | Compilers/Named/ContextProperties | 0m03.00s || -0m00.02s | -0.66% 0m02.90s | Compilers/TestCase | 0m02.89s || +0m00.00s | +0.34% 0m02.88s | LegacyArithmetic/ZBoundedZ | 0m03.85s || -0m00.97s | -25.19% 0m02.88s | Util/WordUtil | 0m02.90s || -0m00.02s | -0.68% 0m02.72s | Compilers/Named/CompileInterp | 0m02.74s || -0m00.02s | -0.72% 0m02.58s | Arithmetic/Saturated/Freeze | 0m02.56s || +0m00.02s | +0.78% 0m02.58s | LegacyArithmetic/BarretReduction | 0m02.72s || -0m00.14s | -5.14% 0m02.54s | Compilers/Named/ContextProperties/Proper | 0m02.61s || -0m00.06s | -2.68% 0m02.40s | Arithmetic/ModularArithmeticTheorems | 0m03.33s || -0m00.93s | -27.92% 0m02.38s | Specific/NISTP256/FancyMachine256/Montgomery | 0m02.33s || +0m00.04s | +2.14% 0m02.30s | Specific/NISTP256/FancyMachine256/Core | 0m02.28s || +0m00.02s | +0.87% 0m02.27s | Compilers/CommonSubexpressionEliminationProperties | 0m02.20s || +0m00.06s | +3.18% 0m02.22s | Compilers/Z/Bounds/Relax | 0m02.21s || +0m00.01s | +0.45% 0m02.22s | Specific/NISTP256/FancyMachine256/Barrett | 0m02.27s || -0m00.04s | -2.20% 0m02.16s | Util/ZUtil/Quot | 0m02.08s || +0m00.08s | +3.84% 0m02.10s | Compilers/Named/NameUtilProperties | 0m02.04s || +0m00.06s | +2.94% 0m02.10s | Compilers/Z/RewriteAddToAdcInterp | 0m02.14s || -0m00.04s | -1.86% 0m02.10s | p224_32.c | 0m02.11s || -0m00.00s | -0.47% 0m02.09s | Specific/Framework/ArithmeticSynthesis/Defaults | 0m02.11s || -0m00.02s | -0.94% 0m02.07s | Util/ZRange/SplitBounds | 0m02.01s || +0m00.06s | +2.98% 0m02.01s | curve25519_32.c | 0m02.02s || -0m00.01s | -0.49% 0m01.90s | Compilers/Z/JavaNotations | 0m01.96s || -0m00.06s | -3.06% 0m01.84s | LegacyArithmetic/MontgomeryReduction | 0m01.82s || +0m00.02s | +1.09% 0m01.84s | Util/ZUtil/AddGetCarry | 0m01.87s || -0m00.03s | -1.60% 0m01.73s | Util/ZUtil/Pow2Mod | 0m01.48s || +0m00.25s | +16.89% 0m01.68s | Compilers/Named/WfFromUnit | 0m01.70s || -0m00.02s | -1.17% 0m01.67s | Util/Tuple | 0m01.63s || +0m00.04s | +2.45% 0m01.66s | Arithmetic/CoreUnfolder | 0m01.66s || +0m00.00s | +0.00% 0m01.64s | secp256k1_64.c | 0m01.50s || +0m00.13s | +9.33% 0m01.63s | p256_64.c | 0m01.53s || +0m00.09s | +6.53% 0m01.56s | Specific/Framework/ReificationTypes | 0m01.71s || -0m00.14s | -8.77% 0m01.53s | p224_64.c | 0m01.52s || +0m00.01s | +0.65% 0m01.52s | Specific/Framework/ArithmeticSynthesis/Base | 0m01.49s || +0m00.03s | +2.01% 0m01.50s | Compilers/Relations | 0m01.48s || +0m00.02s | +1.35% 0m01.47s | Specific/Framework/OutputType | 0m01.48s || -0m00.01s | -0.67% 0m01.45s | Compilers/Named/InterpretToPHOASWf | 0m01.48s || -0m00.03s | -2.02% 0m01.45s | Experiments/NewPipeline/CLI | 0m01.41s || +0m00.04s | +2.83% 0m01.40s | LegacyArithmetic/Double/Proofs/BitwiseOr | 0m01.28s || +0m00.11s | +9.37% 0m01.39s | curve25519_64.c | 0m01.38s || +0m00.01s | +0.72% 0m01.37s | Arithmetic/PrimeFieldTheorems | 0m01.30s || +0m00.07s | +5.38% 0m01.32s | Curves/Edwards/XYZT/Precomputed | 0m01.28s || +0m00.04s | +3.12% 0m01.30s | Specific/Framework/ArithmeticSynthesis/Karatsuba | 0m01.34s || -0m00.04s | -2.98% 0m01.28s | Util/QUtil | 0m01.52s || -0m00.24s | -15.78% 0m01.25s | Util/ZUtil/Testbit | 0m01.06s || +0m00.18s | +17.92% 0m01.23s | Experiments/NewPipeline/StandaloneOCamlMain | 0m01.23s || +0m00.00s | +0.00% 0m01.22s | Arithmetic/Saturated/CoreUnfolder | 0m01.12s || +0m00.09s | +8.92% 0m01.20s | Experiments/NewPipeline/Language | 0m01.22s || -0m00.02s | -1.63% 0m01.20s | Experiments/NewPipeline/StandaloneHaskellMain | 0m01.30s || -0m00.10s | -7.69% 0m01.19s | LegacyArithmetic/Double/Proofs/LoadImmediate | 0m01.40s || -0m00.20s | -15.00% 0m01.18s | LegacyArithmetic/BaseSystemProofs | 0m01.24s || -0m00.06s | -4.83% 0m01.18s | Util/ZRange/BasicLemmas | 0m01.18s || +0m00.00s | +0.00% 0m01.17s | Compilers/LinearizeInterp | 0m01.19s || -0m00.02s | -1.68% 0m01.17s | Experiments/NewPipeline/CompilersTestCases | 0m01.07s || +0m00.09s | +9.34% 0m01.14s | Compilers/Z/Syntax/Util | 0m00.84s || +0m00.29s | +35.71% 0m01.11s | Compilers/MultiSizeTest | 0m01.13s || -0m00.01s | -1.76% 0m01.08s | Compilers/Z/RewriteAddToAdcWf | 0m01.08s || +0m00.00s | +0.00% 0m01.06s | Experiments/NewPipeline/AbstractInterpretation | 0m01.07s || -0m00.01s | -0.93% 0m01.00s | Experiments/NewPipeline/RewriterProofs | 0m00.90s || +0m00.09s | +11.11% 0m01.00s | Specific/X25519/C32/CurveParameters | 0m00.95s || +0m00.05s | +5.26% 0m00.96s | Arithmetic/Saturated/WrappersUnfolder | 0m01.08s || -0m00.12s | -11.11% 0m00.96s | Compilers/Named/InterpretToPHOASInterp | 0m01.02s || -0m00.06s | -5.88% 0m00.96s | Specific/Framework/SynthesisFramework | 0m01.10s || -0m00.14s | -12.72% 0m00.95s | Util/ZUtil/Stabilization | 0m01.02s || -0m00.07s | -6.86% 0m00.92s | Specific/Framework/IntegrationTestDisplayCommon | 0m00.98s || -0m00.05s | -6.12% 0m00.90s | Compilers/Z/Bounds/Pipeline/ReflectiveTactics | 0m00.88s || +0m00.02s | +2.27% 0m00.89s | Compilers/Z/CommonSubexpressionElimination | 0m00.98s || -0m00.08s | -9.18% 0m00.89s | Util/NumTheoryUtil | 0m01.21s || -0m00.31s | -26.44% 0m00.86s | Arithmetic/Saturated/FreezeUnfolder | 0m00.80s || +0m00.05s | +7.49% 0m00.86s | Compilers/Named/FMapContext | 0m00.82s || +0m00.04s | +4.87% 0m00.85s | Arithmetic/Saturated/UniformWeight | 0m00.93s || -0m00.08s | -8.60% 0m00.84s | Specific/Framework/ArithmeticSynthesis/Freeze | 0m00.89s || -0m00.05s | -5.61% 0m00.82s | Compilers/Named/CompileProperties | 0m00.84s || -0m00.02s | -2.38% 0m00.82s | Compilers/Named/InterpSideConditionsInterp | 0m00.80s || +0m00.01s | +2.49% 0m00.82s | Specific/Framework/ArithmeticSynthesis/MontgomeryPackage | 0m00.83s || -0m00.01s | -1.20% 0m00.82s | Util/CPSUtil | 0m00.72s || +0m00.09s | +13.88% 0m00.81s | Compilers/InlineConstAndOpInterp | 0m00.79s || +0m00.02s | +2.53% 0m00.81s | Util/ZUtil/CC | 0m00.74s || +0m00.07s | +9.45% 0m00.80s | Compilers/InterpByIsoProofs | 0m00.84s || -0m00.03s | -4.76% 0m00.80s | Util/ZUtil/Log2 | N/A || +0m00.80s | ∞ 0m00.79s | Specific/Framework/IntegrationTestTemporaryMiscCommon | 0m00.76s || +0m00.03s | +3.94% 0m00.78s | Arithmetic/Saturated/MulSplitUnfolder | 0m00.91s || -0m00.13s | -14.28% 0m00.76s | Compilers/Named/AListContext | 0m01.10s || -0m00.34s | -30.90% 0m00.76s | Util/ZUtil/Divide | N/A || +0m00.76s | ∞ 0m00.75s | Specific/Framework/ArithmeticSynthesis/SquareFromMul | 0m00.71s || +0m00.04s | +5.63% 0m00.75s | Util/ZUtil/EquivModulo | 0m00.68s || +0m00.06s | +10.29% 0m00.74s | Compilers/MapCastByDeBruijnInterp | 0m00.86s || -0m00.12s | -13.95% 0m00.74s | Specific/Framework/ArithmeticSynthesis/LadderstepPackage | 0m00.72s || +0m00.02s | +2.77% 0m00.74s | Specific/Framework/MontgomeryReificationTypesPackage | 0m00.71s || +0m00.03s | +4.22% 0m00.73s | Arithmetic/MontgomeryReduction/WordByWord/Definition | 0m00.77s || -0m00.04s | -5.19% 0m00.73s | Util/ZUtil/Tactics/RewriteModSmall | 0m00.80s || -0m00.07s | -8.75% 0m00.72s | Specific/Framework/ReificationTypesPackage | 0m00.75s || -0m00.03s | -4.00% 0m00.72s | Util/ZUtil/Le | 0m00.30s || +0m00.42s | +140.00% 0m00.72s | Util/ZUtil/Rshi | 0m00.74s || -0m00.02s | -2.70% 0m00.72s | Util/ZUtil/Z2Nat | 0m00.31s || +0m00.41s | +132.25% 0m00.71s | Compilers/Z/Bounds/Pipeline | 0m00.66s || +0m00.04s | +7.57% 0m00.70s | Experiments/NewPipeline/MiscCompilerPasses | 0m00.70s || +0m00.00s | +0.00% 0m00.70s | Specific/Framework/MontgomeryReificationTypes | 0m00.75s || -0m00.05s | -6.66% 0m00.69s | Compilers/CommonSubexpressionEliminationInterp | 0m00.66s || +0m00.02s | +4.54% 0m00.69s | Specific/Framework/ArithmeticSynthesis/DefaultsPackage | 0m00.74s || -0m00.05s | -6.75% 0m00.69s | Specific/Framework/ArithmeticSynthesis/HelperTactics | 0m00.69s || +0m00.00s | +0.00% 0m00.69s | Specific/Framework/ArithmeticSynthesis/KaratsubaPackage | 0m00.68s || +0m00.00s | +1.47% 0m00.68s | Arithmetic/Saturated/Wrappers | 0m00.70s || -0m00.01s | -2.85% 0m00.68s | Specific/Framework/ArithmeticSynthesis/BasePackage | 0m00.72s || -0m00.03s | -5.55% 0m00.68s | Specific/Framework/ArithmeticSynthesis/FreezePackage | 0m00.72s || -0m00.03s | -5.55% 0m00.68s | Specific/Framework/ArithmeticSynthesis/Ladderstep | 0m00.72s || -0m00.03s | -5.55% 0m00.67s | Arithmetic/Saturated/UniformWeightInstances | 0m00.68s || -0m00.01s | -1.47% 0m00.67s | Compilers/SmartMap | 0m00.70s || -0m00.02s | -4.28% 0m00.67s | LegacyArithmetic/Double/Proofs/SelectConditional | 0m00.69s || -0m00.01s | -2.89% 0m00.65s | Compilers/CommonSubexpressionElimination | 0m00.65s || +0m00.00s | +0.00% 0m00.63s | Compilers/MapCastByDeBruijnWf | 0m00.63s || +0m00.00s | +0.00% 0m00.62s | LegacyArithmetic/Interface | 0m00.74s || -0m00.12s | -16.21% 0m00.61s | Compilers/Named/WfInterp | 0m00.58s || +0m00.03s | +5.17% 0m00.60s | Compilers/InputSyntax | 0m00.50s || +0m00.09s | +19.99% 0m00.60s | Compilers/MapBaseTypeWf | 0m00.58s || +0m00.02s | +3.44% 0m00.60s | Compilers/Z/Bounds/MapCastByDeBruijnWf | 0m00.53s || +0m00.06s | +13.20% 0m00.60s | Compilers/Z/Bounds/Pipeline/Glue | 0m00.61s || -0m00.01s | -1.63% 0m00.60s | Util/NUtil | 0m00.69s || -0m00.08s | -13.04% 0m00.60s | Util/ZUtil/Lnot | N/A || +0m00.60s | ∞ 0m00.60s | Util/ZUtil/Mul | N/A || +0m00.60s | ∞ 0m00.59s | Compilers/Z/Bounds/MapCastByDeBruijnInterp | 0m00.59s || +0m00.00s | +0.00% 0m00.58s | Compilers/InterpWfRel | 0m00.52s || +0m00.05s | +11.53% 0m00.58s | Compilers/Z/Bounds/RoundUpLemmas | 0m00.52s || +0m00.05s | +11.53% 0m00.58s | Compilers/Z/Reify | 0m00.60s || -0m00.02s | -3.33% 0m00.58s | LegacyArithmetic/Double/Core | 0m00.58s || +0m00.00s | +0.00% 0m00.58s | Spec/EdDSA | 0m00.60s || -0m00.02s | -3.33% 0m00.57s | Arithmetic/ModularArithmeticPre | 0m00.60s || -0m00.03s | -5.00% 0m00.57s | Compilers/Z/Named/RewriteAddToAdc | 0m00.69s || -0m00.12s | -17.39% 0m00.56s | Compilers/Z/Bounds/InterpretationLemmas/Tactics | 0m00.60s || -0m00.03s | -6.66% 0m00.56s | Util/HList | 0m00.50s || +0m00.06s | +12.00% 0m00.55s | Compilers/Z/FoldTypes | 0m00.48s || +0m00.07s | +14.58% 0m00.52s | Compilers/Z/MapCastByDeBruijnInterp | 0m00.55s || -0m00.03s | -5.45% 0m00.52s | Compilers/Z/Syntax | 0m00.52s || +0m00.00s | +0.00% 0m00.52s | Util/Decidable/Decidable2Bool | 0m00.53s || -0m00.01s | -1.88% 0m00.52s | Util/ZBounded | 0m00.46s || +0m00.06s | +13.04% 0m00.51s | Compilers/Z/Bounds/Interpretation | 0m00.50s || +0m00.01s | +2.00% 0m00.50s | Compilers/GeneralizeVarInterp | 0m00.48s || +0m00.02s | +4.16% 0m00.50s | Compilers/Z/CommonSubexpressionEliminationWf | 0m00.56s || -0m00.06s | -10.71% 0m00.50s | Compilers/Z/RewriteAddToAdc | 0m00.65s || -0m00.15s | -23.07% 0m00.50s | LegacyArithmetic/ArchitectureToZLike | 0m00.51s || -0m00.01s | -1.96% 0m00.49s | Compilers/GeneralizeVarWf | 0m00.49s || +0m00.00s | +0.00% 0m00.49s | Compilers/InlineConstAndOpByRewriteWf | 0m00.51s || -0m00.02s | -3.92% 0m00.49s | Compilers/Z/ArithmeticSimplifierUtil | 0m00.50s || -0m00.01s | -2.00% 0m00.49s | Compilers/Z/InlineInterp | 0m00.54s || -0m00.05s | -9.25% 0m00.49s | Compilers/Z/InlineWf | 0m00.49s || +0m00.00s | +0.00% 0m00.48s | Compilers/Reify | 0m00.46s || +0m00.01s | +4.34% 0m00.48s | Compilers/Z/Bounds/MapCastByDeBruijn | 0m00.53s || -0m00.05s | -9.43% 0m00.48s | Compilers/Z/GeneralizeVarInterp | 0m00.46s || +0m00.01s | +4.34% 0m00.48s | Compilers/Z/InlineConstAndOpByRewrite | 0m00.51s || -0m00.03s | -5.88% 0m00.48s | Compilers/Z/InlineConstAndOpByRewriteInterp | 0m00.46s || +0m00.01s | +4.34% 0m00.48s | Compilers/Z/InlineConstAndOpInterp | 0m00.50s || -0m00.02s | -4.00% 0m00.48s | Experiments/NewPipeline/UnderLets | 0m00.46s || +0m00.01s | +4.34% 0m00.47s | Compilers/InterpWf | 0m00.49s || -0m00.02s | -4.08% 0m00.47s | Compilers/Named/PositiveContext/DefaultsProperties | 0m00.45s || +0m00.01s | +4.44% 0m00.47s | Compilers/Z/InterpSideConditions | 0m00.51s || -0m00.04s | -7.84% 0m00.46s | Compilers/InterpProofs | 0m00.44s || +0m00.02s | +4.54% 0m00.46s | Compilers/Named/DeadCodeEliminationInterp | 0m00.50s || -0m00.03s | -7.99% 0m00.46s | Compilers/Z/CommonSubexpressionEliminationInterp | 0m00.56s || -0m00.10s | -17.85% 0m00.46s | Compilers/Z/InlineConstAndOp | 0m00.50s || -0m00.03s | -7.99% 0m00.46s | Compilers/Z/MapCastByDeBruijn | 0m00.43s || +0m00.03s | +6.97% 0m00.46s | LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic | 0m00.58s || -0m00.11s | -20.68% 0m00.46s | Specific/Framework/CurveParameters | 0m00.45s || +0m00.01s | +2.22% 0m00.45s | Compilers/Z/Inline | 0m00.55s || -0m00.10s | -18.18% 0m00.45s | Specific/X25519/C64/CurveParameters | 0m00.44s || +0m00.01s | +2.27% 0m00.44s | Compilers/InlineConstAndOpByRewriteInterp | 0m00.48s || -0m00.03s | -8.33% 0m00.44s | Compilers/Z/MapCastByDeBruijnWf | 0m00.57s || -0m00.12s | -22.80% 0m00.44s | Compilers/ZExtended/Syntax | 0m00.42s || +0m00.02s | +4.76% 0m00.44s | LegacyArithmetic/BaseSystem | 0m00.60s || -0m00.15s | -26.66% 0m00.44s | Util/ZRange | 0m00.44s || +0m00.00s | +0.00% 0m00.43s | Compilers/Named/WeakListContext | 0m00.44s || -0m00.01s | -2.27% 0m00.43s | Compilers/ZExtended/MapBaseType | 0m00.44s || -0m00.01s | -2.27% 0m00.43s | Specific/Framework/IntegrationTestDisplayCommonTactics | 0m00.49s || -0m00.06s | -12.24% 0m00.43s | Util/NUtil/WithoutReferenceToZ | N/A || +0m00.43s | ∞ 0m00.43s | Util/ZUtil/CPS | 0m00.44s || -0m00.01s | -2.27% 0m00.42s | Compilers/Named/InterpSideConditions | 0m00.32s || +0m00.09s | +31.24% 0m00.42s | Compilers/Z/GeneralizeVar | 0m00.39s || +0m00.02s | +7.69% 0m00.42s | Compilers/Z/GeneralizeVarWf | 0m00.46s || -0m00.04s | -8.69% 0m00.42s | Compilers/Z/InlineConstAndOpWf | 0m00.54s || -0m00.12s | -22.22% 0m00.42s | Compilers/Z/Named/DeadCodeEliminationInterp | 0m00.46s || -0m00.04s | -8.69% 0m00.42s | LegacyArithmetic/ZBounded | 0m00.59s || -0m00.17s | -28.81% 0m00.42s | Specific/Framework/RawCurveParameters | 0m00.41s || +0m00.01s | +2.43% 0m00.42s | Util/ZRange/Operations | 0m00.52s || -0m00.10s | -19.23% 0m00.41s | Compilers/Z/TypeInversion | 0m00.36s || +0m00.04s | +13.88% 0m00.40s | Compilers/GeneralizeVar | 0m00.35s || +0m00.05s | +14.28% 0m00.40s | Compilers/InlineConstAndOp | 0m00.39s || +0m00.01s | +2.56% 0m00.40s | Compilers/Z/InlineConstAndOpByRewriteWf | 0m00.49s || -0m00.08s | -18.36% 0m00.39s | Compilers/Named/RegisterAssign | 0m00.36s || +0m00.03s | +8.33% 0m00.38s | Compilers/Inline | 0m00.39s || -0m00.01s | -2.56% 0m00.38s | Compilers/Named/Wf | 0m00.37s || +0m00.01s | +2.70% 0m00.38s | Compilers/StripExpr | 0m00.33s || +0m00.04s | +15.15% 0m00.38s | Compilers/Z/Named/DeadCodeElimination | 0m00.35s || +0m00.03s | +8.57% 0m00.38s | Specific/Framework/CurveParametersPackage | 0m00.34s || +0m00.03s | +11.76% 0m00.38s | Specific/NISTP256/AMD128/CurveParameters | 0m00.36s || +0m00.02s | +5.55% 0m00.38s | Specific/NISTP256/AMD64/CurveParameters | 0m00.40s || -0m00.02s | -5.00% 0m00.38s | Specific/X2448/Karatsuba/C64/CurveParameters | 0m00.36s || +0m00.02s | +5.55% 0m00.38s | Util/ZUtil/Definitions | 0m00.29s || +0m00.09s | +31.03% 0m00.37s | Compilers/Z/Bounds/Pipeline/OutputType | 0m00.35s || +0m00.02s | +5.71% 0m00.36s | Compilers/Named/Compile | 0m00.34s || +0m00.01s | +5.88% 0m00.36s | Compilers/Named/ContextProperties/Tactics | 0m00.38s || -0m00.02s | -5.26% 0m00.36s | Compilers/Named/DeadCodeElimination | 0m00.36s || +0m00.00s | +0.00% 0m00.36s | Compilers/Named/EstablishLiveness | 0m00.36s || +0m00.00s | +0.00% 0m00.36s | Compilers/Named/GetNames | 0m00.35s || +0m00.01s | +2.85% 0m00.36s | Compilers/Named/MapCast | 0m00.36s || +0m00.00s | +0.00% 0m00.36s | Util/ZUtil/Tactics/SimplifyFractionsLe | 0m00.31s || +0m00.04s | +16.12% 0m00.36s | Util/ZUtil/Tactics/ZeroBounds | 0m00.35s || +0m00.01s | +2.85% 0m00.35s | Compilers/Named/ContextOn | 0m00.33s || +0m00.01s | +6.06% 0m00.35s | Compilers/Named/PositiveContext/Defaults | 0m00.42s || -0m00.07s | -16.66% 0m00.35s | Compilers/ZExtended/InlineConstAndOpInterp | 0m00.35s || +0m00.00s | +0.00% 0m00.35s | Compilers/ZExtended/Syntax/Util | 0m00.37s || -0m00.02s | -5.40% 0m00.35s | LegacyArithmetic/Pow2Base | 0m00.46s || -0m00.11s | -23.91% 0m00.35s | Util/ZUtil/Odd | N/A || +0m00.35s | ∞ 0m00.35s | Util/ZUtil/Pow | N/A || +0m00.35s | ∞ 0m00.35s | Util/ZUtil/Pow2 | N/A || +0m00.35s | ∞ 0m00.34s | Compilers/InlineConstAndOpByRewrite | 0m00.35s || -0m00.00s | -2.85% 0m00.34s | Compilers/Named/CountLets | 0m00.34s || +0m00.00s | +0.00% 0m00.34s | Compilers/Named/MapType | 0m00.34s || +0m00.00s | +0.00% 0m00.34s | Compilers/Named/PositiveContext | 0m00.38s || -0m00.03s | -10.52% 0m00.34s | Compilers/Named/Syntax | 0m00.34s || +0m00.00s | +0.00% 0m00.34s | Compilers/Tuple | 0m00.34s || +0m00.00s | +0.00% 0m00.34s | Compilers/ZExtended/InlineConstAndOpByRewriteInterp | 0m00.35s || -0m00.00s | -2.85% 0m00.34s | Compilers/ZExtended/InlineConstAndOpWf | 0m00.34s || +0m00.00s | +0.00% 0m00.34s | Util/ZUtil/Land | 0m00.29s || +0m00.05s | +17.24% 0m00.34s | Util/ZUtil/N2Z | N/A || +0m00.34s | ∞ 0m00.34s | Util/ZUtil/Tactics/PullPush/Modulo | 0m00.33s || +0m00.01s | +3.03% 0m00.34s | Util/ZUtil/Tactics/Ztestbit | 0m00.36s || -0m00.01s | -5.55% 0m00.33s | Arithmetic/MontgomeryReduction/Definition | 0m00.52s || -0m00.19s | -36.53% 0m00.33s | Compilers/CountLets | 0m00.30s || +0m00.03s | +10.00% 0m00.33s | Compilers/FoldTypes | 0m00.31s || +0m00.02s | +6.45% 0m00.33s | Compilers/InterpByIso | 0m00.35s || -0m00.01s | -5.71% 0m00.33s | Compilers/MapCastByDeBruijn | 0m00.60s || -0m00.26s | -44.99% 0m00.33s | Compilers/Named/ContextDefinitions | 0m00.36s || -0m00.02s | -8.33% 0m00.33s | Compilers/Named/SmartMap | 0m00.32s || +0m00.01s | +3.12% 0m00.33s | Util/BoundedWord | 0m00.43s || -0m00.09s | -23.25% 0m00.33s | Util/ZUtil/Hints | 0m00.33s || +0m00.00s | +0.00% 0m00.33s | Util/ZUtil/Hints/ZArith | 0m00.33s || +0m00.00s | +0.00% 0m00.32s | Compilers/FilterLive | 0m00.35s || -0m00.02s | -8.57% 0m00.32s | Compilers/MapBaseType | 0m00.32s || +0m00.00s | +0.00% 0m00.32s | Compilers/Named/ExprInversion | 0m00.34s || -0m00.02s | -5.88% 0m00.32s | Compilers/Named/IdContext | 0m00.31s || +0m00.01s | +3.22% 0m00.32s | Compilers/Named/InterpretToPHOAS | 0m00.35s || -0m00.02s | -8.57% 0m00.32s | Compilers/ZExtended/InlineConstAndOp | 0m00.34s || -0m00.02s | -5.88% 0m00.32s | Util/IdfunWithAlt | 0m00.32s || +0m00.00s | +0.00% 0m00.32s | Util/ZRange/Show | 0m00.32s || +0m00.00s | +0.00% 0m00.32s | Util/ZUtil/DistrIf | N/A || +0m00.32s | ∞ 0m00.32s | Util/ZUtil/Opp | N/A || +0m00.32s | ∞ 0m00.31s | Compilers/CommonSubexpressionEliminationDenote | 0m00.38s || -0m00.07s | -18.42% 0m00.31s | Compilers/Linearize | 0m00.34s || -0m00.03s | -8.82% 0m00.31s | Compilers/Named/Context | 0m00.34s || -0m00.03s | -8.82% 0m00.31s | Spec/ModularArithmetic | 0m00.41s || -0m00.09s | -24.39% 0m00.31s | Util/ZUtil/Tactics | 0m00.29s || +0m00.02s | +6.89% 0m00.30s | Compilers/Z/OpInversion | 0m00.35s || -0m00.04s | -14.28% 0m00.30s | Compilers/ZExtended/InlineConstAndOpByRewrite | 0m00.34s || -0m00.04s | -11.76% 0m00.30s | Compilers/ZExtended/InlineConstAndOpByRewriteWf | 0m00.33s || -0m00.03s | -9.09% 0m00.30s | Util/ZUtil/MulSplit | 0m00.37s || -0m00.07s | -18.91% 0m00.28s | Arithmetic/MontgomeryReduction/WordByWord/Abstract/Definition | 0m00.26s || +0m00.02s | +7.69% 0m00.27s | Util/ZUtil/AddModulo | 0m00.25s || +0m00.02s | +8.00% 0m00.27s | Util/ZUtil/Tactics/PullPush | 0m00.26s || +0m00.01s | +3.84% 0m00.25s | Arithmetic/MontgomeryReduction/WordByWord/Abstract/Dependent/Definition | 0m00.24s || +0m00.01s | +4.16% 0m00.24s | Util/ZUtil/Zselect | 0m00.25s || -0m00.01s | -4.00%
* git submodule update --remote --recursiveGravatar Andres Erbsen2018-02-24
|
* minor updates needed to make it compile with bbvGravatar Samuel Gruetter2018-02-05
| | | | removing lemma wordToNat_wzero is ok because it's already in bbv
* 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).
* Split off notation and defs in ZUtilGravatar Jason Gross2017-05-12
|
* s/appcontext/context/Gravatar Jason Gross2017-05-11
| | | | They mean the same thing since 8.5, and appcontext is deprecated.
* Add wordToZ_ZToWord_modGravatar Jason Gross2017-04-08
|
* Add ZToWord_wordToZ_ZToWord_smallGravatar Jason Gross2017-04-08
|
* More fine-grained tactic importsGravatar Jason Gross2017-04-03
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Most files no longer import Crypto.Util.Tactics. We remove an unused lemma depending on classical axioms; closes #143. After | File Name | Before || Change ----------------------------------------------------------------------------------------------------------- 28m38.18s | Total | 29m04.51s || -0m26.32s ----------------------------------------------------------------------------------------------------------- 0m41.70s | ModularArithmetic/ModularBaseSystemProofs | 0m32.66s || +0m09.04s 1m39.88s | MontgomeryX | 1m46.07s || -0m06.18s 1m56.52s | WeierstrassCurve/Projective | 2m00.76s || -0m04.23s 10m36.85s | WeierstrassCurve/WeierstrassCurveTheorems | 10m40.14s || -0m03.28s 0m21.35s | ModularArithmetic/Pow2BaseProofs | 0m22.54s || -0m01.18s 0m20.24s | Reflection/Named/MapCastWf | 0m21.41s || -0m01.17s 1m30.28s | Test/Curve25519SpecTestVectors | 1m31.19s || -0m00.90s 0m49.53s | Specific/IntegrationTest | 0m50.01s || -0m00.47s 0m42.19s | MontgomeryCurveTheorems | 0m42.18s || +0m00.00s 0m41.08s | ModularArithmetic/Conversion | 0m41.84s || -0m00.76s 0m36.62s | Spec/Ed25519 | 0m37.13s || -0m00.51s 0m23.64s | CompleteEdwardsCurve/CompleteEdwardsCurveTheorems | 0m24.44s || -0m00.80s 0m19.94s | Specific/GF25519 | 0m20.12s || -0m00.17s 0m19.59s | CompleteEdwardsCurve/ExtendedCoordinates | 0m19.83s || -0m00.23s 0m19.14s | Reflection/Z/Bounds/InterpretationLemmas | 0m19.90s || -0m00.75s 0m18.65s | EdDSARepChange | 0m18.74s || -0m00.08s 0m16.24s | Reflection/Z/ArithmeticSimplifierWf | 0m17.11s || -0m00.87s 0m15.03s | Util/ZUtil | 0m15.93s || -0m00.90s 0m14.74s | Reflection/Named/ContextProperties/NameUtil | 0m15.11s || -0m00.36s 0m14.62s | Reflection/Named/ContextProperties/SmartMap | 0m14.93s || -0m00.31s 0m12.96s | Specific/NewBaseSystemTest | 0m13.24s || -0m00.27s 0m11.84s | Algebra/Field | 0m12.49s || -0m00.65s 0m10.21s | Testbit | 0m09.86s || +0m00.35s 0m09.86s | Reflection/Z/ArithmeticSimplifierInterp | 0m10.69s || -0m00.83s 0m09.44s | Reflection/Named/MapCastInterp | 0m09.82s || -0m00.38s 0m08.81s | BoundedArithmetic/ArchitectureToZLikeProofs | 0m09.37s || -0m00.55s 0m08.60s | Assembly/GF25519 | 0m08.66s || -0m00.06s 0m08.58s | ModularArithmetic/Montgomery/ZProofs | 0m08.77s || -0m00.18s 0m08.53s | BoundedArithmetic/Double/Proofs/ShiftRightDoubleWordImmediate | 0m08.34s || +0m00.18s 0m08.41s | BoundedArithmetic/Double/Proofs/Multiply | 0m08.77s || -0m00.35s 0m08.26s | Reflection/InlineWf | 0m08.59s || -0m00.33s 0m07.54s | Algebra/Ring | 0m08.04s || -0m00.49s 0m07.43s | MxDHRepChange | 0m07.10s || +0m00.33s 0m07.15s | BoundedArithmetic/Double/Proofs/SpreadLeftImmediate | 0m07.09s || +0m00.06s 0m07.00s | NewBaseSystem | 0m07.16s || -0m00.16s 0m06.51s | Specific/GF1305 | 0m06.52s || -0m00.00s 0m06.09s | Util/FixedWordSizesEquality | 0m06.37s || -0m00.28s 0m05.56s | BoundedArithmetic/Double/Proofs/RippleCarryAddSub | 0m05.51s || +0m00.04s 0m05.38s | CompleteEdwardsCurve/Pre | 0m05.38s || +0m00.00s 0m05.28s | ModularArithmetic/ModularBaseSystemListProofs | 0m05.15s || +0m00.12s 0m05.24s | Experiments/GenericFieldPow | 0m05.54s || -0m00.29s 0m05.01s | Specific/SC25519 | 0m05.38s || -0m00.37s 0m04.93s | Algebra/Field_test | 0m04.81s || +0m00.12s 0m04.78s | Reflection/InlineCastWf | 0m04.94s || -0m00.16s 0m04.10s | Reflection/Z/Syntax/Equality | 0m04.28s || -0m00.18s 0m03.92s | BaseSystemProofs | 0m03.90s || +0m00.02s 0m03.75s | ModularArithmetic/BarrettReduction/ZHandbook | 0m03.94s || -0m00.18s 0m03.72s | CompleteEdwardsCurve/EdwardsMontgomery | 0m03.69s || +0m00.03s 0m03.72s | Reflection/EtaWf | 0m03.71s || +0m00.01s 0m03.60s | Reflection/Named/CompileWf | 0m04.01s || -0m00.40s 0m03.58s | SaturatedBaseSystem | 0m03.76s || -0m00.17s 0m03.33s | BoundedArithmetic/InterfaceProofs | 0m03.72s || -0m00.39s 0m03.16s | Reflection/LinearizeWf | 0m03.26s || -0m00.09s 0m03.08s | ModularArithmetic/ZBoundedZ | 0m03.16s || -0m00.08s 0m03.01s | Specific/FancyMachine256/Montgomery | 0m03.16s || -0m00.15s 0m02.99s | Reflection/Named/CompileInterp | 0m03.24s || -0m00.25s 0m02.92s | ModularArithmetic/ModularArithmeticTheorems | 0m03.06s || -0m00.14s 0m02.92s | ModularArithmetic/BarrettReduction/ZGeneralized | 0m03.15s || -0m00.23s 0m02.90s | Specific/FancyMachine256/Barrett | 0m03.18s || -0m00.28s 0m02.80s | Spec/MontgomeryCurve | 0m03.05s || -0m00.25s 0m02.77s | BoundedArithmetic/Double/Proofs/ShiftRight | 0m02.75s || +0m00.02s 0m02.75s | BoundedArithmetic/Double/Proofs/Decode | 0m02.81s || -0m00.06s 0m02.64s | BoundedArithmetic/Double/Proofs/ShiftLeft | 0m02.62s || +0m00.02s 0m02.54s | Reflection/InlineInterp | 0m02.60s || -0m00.06s 0m02.48s | Reflection/Named/ContextProperties | 0m02.58s || -0m00.10s 0m02.47s | ModularArithmetic/ModularBaseSystemOpt | 0m02.39s || +0m00.08s 0m02.40s | Reflection/TestCase | 0m02.60s || -0m00.20s 0m02.35s | ModularArithmetic/BarrettReduction/ZBounded | 0m02.40s || -0m00.04s 0m02.35s | Reflection/Z/Bounds/Relax | 0m02.46s || -0m00.10s 0m02.33s | Reflection/Named/NameUtilProperties | 0m02.40s || -0m00.06s 0m02.15s | Reflection/WfProofs | 0m02.26s || -0m00.10s 0m02.00s | Reflection/WfReflective | 0m02.04s || -0m00.04s 0m01.97s | ModularArithmetic/Montgomery/ZBounded | 0m02.14s || -0m00.17s 0m01.90s | Specific/FancyMachine256/Core | 0m01.98s || -0m00.08s 0m01.89s | Util/WordUtil | 0m01.96s || -0m00.07s 0m01.88s | Assembly/Evaluables | 0m01.82s || +0m00.05s 0m01.62s | WeierstrassCurve/Pre | 0m01.64s || -0m00.01s 0m01.56s | Reflection/Named/InterpretToPHOASWf | 0m01.61s || -0m00.05s 0m01.46s | Assembly/Compile | 0m01.51s || -0m00.05s 0m01.44s | ModularArithmetic/PrimeFieldTheorems | 0m01.43s || +0m00.01s 0m01.44s | ModularArithmetic/BarrettReduction/Z | 0m01.57s || -0m00.13s 0m01.41s | Algebra/Group | 0m01.87s || -0m00.46s 0m01.40s | Util/Tuple | 0m01.46s || -0m00.06s 0m01.38s | Reflection/MapCastInterp | 0m01.38s || +0m00.00s 0m01.31s | BoundedArithmetic/Double/Repeated/Proofs/Decode | 0m01.05s || +0m00.26s 0m01.26s | ModularArithmetic/ExtendedBaseVector | 0m01.28s || -0m00.02s 0m01.16s | Assembly/Conversions | 0m01.13s || +0m00.03s 0m01.14s | Reflection/Z/Bounds/Pipeline/Definition | 0m01.15s || -0m00.01s 0m01.13s | BaseSystem | 0m01.14s || -0m00.01s 0m01.06s | Reflection/SmartBoundInterp | 0m01.07s || -0m00.01s 0m01.04s | Reflection/Named/InterpretToPHOASInterp | 0m00.99s || +0m00.05s 0m01.01s | Reflection/SmartCastWf | 0m00.94s || +0m00.07s 0m01.01s | Assembly/Pipeline | 0m01.02s || -0m00.01s 0m01.01s | Reflection/Relations | 0m01.06s || -0m00.05s 0m00.97s | Assembly/HL | 0m00.99s || -0m00.02s 0m00.96s | Algebra/IntegralDomain | 0m01.00s || -0m00.04s 0m00.94s | Assembly/LL | 0m01.02s || -0m00.08s 0m00.92s | BoundedArithmetic/Double/Proofs/BitwiseOr | 0m00.91s || +0m00.01s 0m00.90s | Assembly/PhoasCommon | 0m00.87s || +0m00.03s 0m00.89s | Util/NumTheoryUtil | 0m00.92s || -0m00.03s 0m00.87s | BoundedArithmetic/Double/Proofs/LoadImmediate | 0m00.96s || -0m00.08s 0m00.84s | Reflection/WfInversion | 0m00.88s || -0m00.04s 0m00.83s | Reflection/InlineCastInterp | 0m00.85s || -0m00.02s 0m00.81s | Reflection/Named/CompileProperties | 0m00.87s || -0m00.05s 0m00.80s | BoundedArithmetic/X86ToZLikeProofs | 0m00.86s || -0m00.05s 0m00.78s | Karatsuba | 0m00.84s || -0m00.05s 0m00.72s | Util/PartiallyReifiedProp | 0m00.73s || -0m00.01s 0m00.72s | Reflection/MultiSizeTest | 0m00.72s || +0m00.00s 0m00.69s | ModularArithmetic/ModularBaseSystem | 0m00.72s || -0m00.03s 0m00.68s | BoundedArithmetic/Double/Repeated/Proofs/Multiply | 0m00.61s || +0m00.07s 0m00.68s | Reflection/MapCastByDeBruijnInterp | 0m00.76s || -0m00.07s 0m00.68s | Encoding/ModularWordEncodingTheorems | 0m00.80s || -0m00.12s 0m00.68s | ModularArithmetic/ExtPow2BaseMulProofs | 0m00.72s || -0m00.03s 0m00.67s | Spec/EdDSA | 0m00.66s || +0m00.01s 0m00.67s | ModularArithmetic/PseudoMersenneBaseParamProofs | 0m00.74s || -0m00.06s 0m00.66s | Reflection/Z/Bounds/Pipeline/ReflectiveTactics | 0m00.62s || +0m00.04s 0m00.66s | Util/IterAssocOp | 0m00.94s || -0m00.27s 0m00.64s | Encoding/ModularWordEncodingPre | 0m00.73s || -0m00.08s 0m00.63s | ModularArithmetic/ModularBaseSystemList | 0m00.77s || -0m00.14s 0m00.62s | Spec/ModularWordEncoding | 0m00.66s || -0m00.04s 0m00.61s | Reflection/MapCastByDeBruijnWf | 0m00.61s || +0m00.00s 0m00.58s | BoundedArithmetic/X86ToZLike | 0m00.57s || +0m00.01s 0m00.58s | Reflection/Z/CNotations | 0m00.56s || +0m00.01s 0m00.57s | Spec/WeierstrassCurve | 0m00.57s || +0m00.00s 0m00.56s | Spec/CompleteEdwardsCurve | 0m00.59s || -0m00.02s 0m00.56s | BoundedArithmetic/Double/Proofs/SelectConditional | 0m00.58s || -0m00.01s 0m00.56s | Reflection/InterpByIsoProofs | 0m00.60s || -0m00.03s 0m00.55s | Reflection/Named/WfInterp | 0m00.57s || -0m00.01s 0m00.55s | BoundedArithmetic/Double/Repeated/Proofs/ShiftLeftRight | 0m00.57s || -0m00.01s 0m00.54s | Reflection/Named/FMapContext | 0m00.70s || -0m00.15s 0m00.54s | Util/AdditionChainExponentiation | 0m00.62s || -0m00.07s 0m00.54s | Reflection/SmartBoundWf | 0m00.55s || -0m00.01s 0m00.54s | Reflection/WfReflectiveGen | 0m00.54s || +0m00.00s 0m00.54s | BoundedArithmetic/Interface | 0m00.56s || -0m00.02s 0m00.52s | BoundedArithmetic/ArchitectureToZLike | 0m00.46s || +0m00.06s 0m00.52s | Reflection/Z/JavaNotations | 0m00.58s || -0m00.05s 0m00.52s | Reflection/Z/Syntax/Util | 0m00.53s || -0m00.01s 0m00.52s | Util/CPSUtil | 0m00.57s || -0m00.04s 0m00.51s | Reflection/BoundByCastInterp | 0m00.51s || +0m00.00s 0m00.50s | BoundedArithmetic/Double/Repeated/Proofs/ShiftRightDoubleWordImmediate | 0m00.53s || -0m00.03s 0m00.50s | BoundedArithmetic/Double/Repeated/Proofs/RippleCarryAddSub | 0m00.57s || -0m00.06s 0m00.50s | Reflection/InterpWfRel | 0m00.54s || -0m00.04s 0m00.49s | Reflection/Z/InlineInterp | 0m00.37s || +0m00.12s 0m00.49s | Reflection/InputSyntax | 0m00.55s || -0m00.06s 0m00.49s | Util/Decidable | 0m00.48s || +0m00.01s 0m00.48s | ModularArithmetic/PseudoMersenneBaseParams | 0m00.39s || +0m00.08s 0m00.48s | BoundedArithmetic/Double/Repeated/Core | 0m00.48s || +0m00.00s 0m00.47s | BoundedArithmetic/Double/Core | 0m00.50s || -0m00.03s 0m00.47s | Reflection/Z/Bounds/Pipeline | 0m00.46s || +0m00.00s 0m00.47s | BoundedArithmetic/Double/Repeated/Proofs/SelectConditional | 0m00.54s || -0m00.07s 0m00.47s | ModularArithmetic/ModularBaseSystemListZOperationsProofs | 0m00.42s || +0m00.04s 0m00.47s | Util/NUtil | 0m00.50s || -0m00.03s 0m00.47s | Reflection/Z/Bounds/Interpretation | 0m00.42s || +0m00.04s 0m00.47s | Reflection/Z/Reify | 0m00.49s || -0m00.02s 0m00.46s | BoundedArithmetic/StripCF | 0m00.44s || +0m00.02s 0m00.46s | BoundedArithmetic/Double/Repeated/Proofs/BitwiseOr | 0m00.51s || -0m00.04s 0m00.46s | Reflection/Z/MapCastByDeBruijn | 0m00.50s || -0m00.03s 0m00.46s | Reflection/Z/Bounds/MapCastByDeBruijnWf | 0m00.42s || +0m00.04s 0m00.46s | BoundedArithmetic/Double/Repeated/Proofs/LoadImmediate | 0m00.55s || -0m00.09s 0m00.45s | Util/HList | 0m00.50s || -0m00.04s 0m00.44s | Reflection/Z/Inline | 0m00.39s || +0m00.04s 0m00.44s | Reflection/InterpWf | 0m00.55s || -0m00.11s 0m00.44s | Reflection/Z/Syntax | 0m00.46s || -0m00.02s 0m00.44s | Reflection/Z/ArithmeticSimplifier | 0m00.47s || -0m00.02s 0m00.44s | Reflection/Named/DeadCodeElimination | 0m00.36s || +0m00.08s 0m00.44s | ModularArithmetic/ZBounded | 0m00.49s || -0m00.04s 0m00.43s | ModularArithmetic/Pre | 0m00.44s || -0m00.01s 0m00.42s | ModularArithmetic/Montgomery/Z | 0m00.39s || +0m00.02s 0m00.42s | Reflection/Z/Bounds/MapCastByDeBruijnInterp | 0m00.43s || -0m00.01s 0m00.42s | Util/ZRange | 0m00.42s || +0m00.00s 0m00.42s | Reflection/Z/MapCastByDeBruijnInterp | 0m00.46s || -0m00.04s 0m00.41s | BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic | 0m00.45s || -0m00.04s 0m00.41s | Reflection/Z/Bounds/MapCastByDeBruijn | 0m00.50s || -0m00.09s 0m00.40s | Reflection/Z/MapCastByDeBruijnWf | 0m00.50s || -0m00.09s 0m00.40s | Reflection/Z/InlineWf | 0m00.42s || -0m00.01s 0m00.40s | Reflection/Z/Bounds/Pipeline/OutputType | 0m00.38s || +0m00.02s 0m00.40s | ModularArithmetic/Pow2Base | 0m00.43s || -0m00.02s 0m00.40s | Reflection/Named/PositiveContext/DefaultsProperties | 0m00.52s || -0m00.12s 0m00.40s | Reflection/MapCastByDeBruijn | 0m00.39s || +0m00.01s 0m00.39s | Reflection/Z/Bounds/Pipeline/Glue | 0m00.46s || -0m00.07s 0m00.39s | Reflection/Named/PositiveContext/Defaults | 0m00.40s || -0m00.01s 0m00.39s | Reflection/Named/ContextDefinitions | 0m00.37s || +0m00.02s 0m00.38s | Reflection/Z/FoldTypes | 0m00.38s || +0m00.00s 0m00.38s | Reflection/Z/HexNotationConstants | 0m00.42s || -0m00.03s 0m00.38s | Reflection/Z/OpInversion | 0m00.37s || +0m00.01s 0m00.38s | ModularArithmetic/ModularBaseSystemListZOperations | 0m00.41s || -0m00.02s 0m00.38s | Reflection/Named/EstablishLiveness | 0m00.38s || +0m00.00s 0m00.38s | Reflection/Named/RegisterAssign | 0m00.38s || +0m00.00s 0m00.38s | Reflection/Reify | 0m00.40s || -0m00.02s 0m00.37s | ModularArithmetic/ModularBaseSystemWord | 0m00.38s || -0m00.01s 0m00.36s | Reflection/Named/InterpretToPHOAS | 0m00.45s || -0m00.09s 0m00.36s | Reflection/Named/Syntax | 0m00.35s || +0m00.01s 0m00.36s | BoundedArithmetic/Eta | 0m00.42s || -0m00.06s 0m00.35s | Reflection/Named/Compile | 0m00.34s || +0m00.00s 0m00.35s | Reflection/MapCastWf | 0m00.31s || +0m00.03s 0m00.35s | Reflection/Named/SmartMap | 0m00.36s || -0m00.01s 0m00.35s | Util/BoundedWord | 0m00.40s || -0m00.05s 0m00.35s | Spec/ModularArithmetic | 0m00.36s || -0m00.01s 0m00.34s | Reflection/Named/ContextOn | 0m00.34s || +0m00.00s 0m00.34s | Reflection/FilterLive | 0m00.32s || +0m00.02s 0m00.34s | Reflection/Named/MapCast | 0m00.37s || -0m00.02s 0m00.33s | Reflection/Named/PositiveContext | 0m00.39s || -0m00.06s 0m00.33s | Algebra/ScalarMult | 0m00.56s || -0m00.23s 0m00.32s | Reflection/Z/BinaryNotationConstants | 0m00.35s || -0m00.02s 0m00.32s | Reflection/Tuple | 0m00.38s || -0m00.06s 0m00.32s | Reflection/Named/ContextProperties/Tactics | 0m00.48s || -0m00.15s 0m00.32s | Reflection/Named/IdContext | 0m00.33s || -0m00.01s 0m00.31s | Reflection/Named/Wf | 0m00.38s || -0m00.07s 0m00.30s | Reflection/MultiSizeTest2 | 0m00.34s || -0m00.04s 0m00.29s | Reflection/ExprInversion | 0m00.26s || +0m00.02s 0m00.29s | Spec/MxDH | 0m00.43s || -0m00.14s 0m00.26s | Algebra/Monoid | 0m00.51s || -0m00.25s 0m00.26s | Util/Sum | 0m00.34s || -0m00.08s 0m00.24s | Algebra | 0m00.43s || -0m00.19s 0m00.23s | Reflection/Equality | 0m00.25s || -0m00.01s 0m00.22s | Reflection/CommonSubexpressionElimination | 0m00.17s || +0m00.04s 0m00.21s | Reflection/SmartMap | 0m00.23s || -0m00.02s 0m00.20s | Reflection/EtaInterp | 0m00.22s || -0m00.01s 0m00.20s | Reflection/BoundByCastWf | 0m00.12s || +0m00.08s 0m00.20s | Reflection/LinearizeInterp | 0m00.23s || -0m00.03s 0m00.18s | Util/LetInMonad | 0m00.19s || -0m00.01s 0m00.16s | Reflection/InterpProofs | 0m00.18s || -0m00.01s 0m00.13s | Util/Option | 0m00.14s || -0m00.01s 0m00.13s | Reflection/Wf | 0m00.12s || +0m00.01s 0m00.12s | Reflection/RewriterWf | 0m00.19s || -0m00.07s 0m00.08s | Reflection/Conversion | 0m00.08s || +0m00.00s 0m00.08s | Reflection/Named/NameUtil | 0m00.12s || -0m00.03s 0m00.07s | Reflection/Inline | 0m00.04s || +0m00.03s 0m00.06s | Reflection/TypeInversion | 0m00.08s || -0m00.02s 0m00.06s | Reflection/SmartBound | 0m00.06s || +0m00.00s 0m00.06s | Reflection/InlineCast | 0m00.06s || +0m00.00s 0m00.06s | Util/Tactics | 0m00.07s || -0m00.01s 0m00.06s | Reflection/RewriterInterp | 0m00.05s || +0m00.00s 0m00.06s | Reflection/MapCast | 0m00.06s || +0m00.00s 0m00.05s | Reflection/TypeUtil | 0m00.04s || +0m00.01s 0m00.04s | Reflection/Syntax | 0m00.09s || -0m00.05s 0m00.04s | Reflection/FoldTypes | 0m00.05s || -0m00.01s 0m00.04s | Reflection/Linearize | 0m00.04s || +0m00.00s 0m00.04s | Reflection/Rewriter | 0m00.03s || +0m00.01s 0m00.04s | Reflection/Map | 0m00.04s || +0m00.00s 0m00.04s | Util/Tactics/OnSubterms | N/A || +0m00.04s 0m00.04s | Reflection/CountLets | 0m00.04s || +0m00.00s 0m00.04s | Reflection/SmartCast | 0m00.04s || +0m00.00s 0m00.04s | Util/LetIn | 0m00.07s || -0m00.03s 0m00.04s | Reflection/Eta | 0m00.05s || -0m00.01s 0m00.04s | Reflection/BoundByCast | 0m00.06s || -0m00.01s 0m00.03s | Reflection/SmartCastInterp | 0m00.05s || -0m00.02s 0m00.03s | Util/Tactics/SubstEvars | N/A || +0m00.03s 0m00.03s | Reflection/InterpByIso | 0m00.04s || -0m00.01s 0m00.03s | Util/Tactics/Forward | N/A || +0m00.03s 0m00.03s | Util/Tactics/BreakMatch | 0m00.02s || +0m00.00s 0m00.03s | Reflection/RenameBinders | 0m00.03s || +0m00.00s 0m00.03s | Util/Tactics/ConvoyDestruct | N/A || +0m00.03s 0m00.02s | Util/Tactics/SideConditionsBeforeToAfter | N/A || +0m00.02s 0m00.02s | Util/Tactics/Revert | N/A || +0m00.02s 0m00.02s | Util/Tactics/Test | N/A || +0m00.02s 0m00.02s | Util/Tactics/SetEvars | N/A || +0m00.02s 0m00.02s | Util/Tactics/SetoidSubst | N/A || +0m00.02s 0m00.02s | Util/Tactics/DestructTrivial | N/A || +0m00.02s 0m00.02s | Util/Tactics/ESpecialize | N/A || +0m00.02s 0m00.02s | Util/Tactics/SimplifyProjections | N/A || +0m00.02s 0m00.02s | Util/Tactics/Not | N/A || +0m00.02s 0m00.02s | Util/Tactics/Contains | N/A || +0m00.02s 0m00.02s | Util/Tactics/SimplifyRepeatedIfs | N/A || +0m00.02s 0m00.02s | Util/Tactics/ClearDuplicates | N/A || +0m00.02s 0m00.02s | Util/Tactics/DebugPrint | N/A || +0m00.02s 0m00.01s | Util/Tactics/GetGoal | N/A || +0m00.01s
* move lemmas from Ed25519 to WordUtilGravatar jadep2017-02-22
|
* Move things from WordUtil to ZUtil, add word lemmaGravatar Jason Gross2017-02-06
|
* More zutilGravatar Jason Gross2017-02-03
|
* Add wordToZ_ZToWord_wordToZGravatar Jason Gross2017-02-01
|
* Add NToWord_wordToN_NToWordGravatar Jason Gross2017-02-01
|
* Add transparent equality proofs for fixed wordTGravatar Jason Gross2017-01-21
| | | | Such a pain to make proofs compute
* Revert "Fix a missing qualification"Gravatar Jason Gross2017-01-21
| | | | | | | | | | This reverts commit 3c4ff8fe8d2154addcf440690d315c58a529c1f6. Revert "Move weqb_hetero to Bedrock.Word" This reverts commit c83cb07f1477de33ce9eb43eea6a4f2720a94763. We probably shouldn't modify Bedrock.Word
* Fix a missing qualificationGravatar Jason Gross2017-01-21
|
* Move weqb_hetero to Bedrock.WordGravatar Jason Gross2017-01-21
|
* Add weqb_heteroGravatar Jason Gross2017-01-21
|
* Lemmas about winit, wlastGravatar Rob Sloan2016-11-11
|
* Fix for Coq 8.4Gravatar Jason Gross2016-11-11
| | | | Tactic notations in sections are automatically local
* Most of the admits in Ed25519.vGravatar Rob Sloan2016-11-11
|
* Fix for 8.4Gravatar Jason Gross2016-11-10
|
* Hint Rewrite is section-local; move to top-levelGravatar Jason Gross2016-11-10
|
* Remove WordizeUtil dependency from WordUtilGravatar Rob Sloan2016-11-09
|
* Rebase + remove WordizeUtil dependency from Z/InterpretationsGravatar Rob Sloan2016-11-09
|\
| * Rewrite cast_word so that it's extracted betterGravatar Jason Gross2016-11-09
| | | | | | | | | | | | | | | | It will now be extracted as the identity function automatically, so we don't need to manually extract it as the empty string. This should also fix #93. (I think the issue was that this was an instance of https://coq.inria.fr/bugs/show_bug.cgi?id=4243.)
* | Finished WordUtil, word operations in Z/InterpretationGravatar Rob Sloan2016-11-09
| |
* | Not quite done with WordUtil lemmas.Gravatar Robert Sloan2016-11-08
|\|
| * put EdDSA encoding sign bit at the MSBGravatar Andres Erbsen2016-11-04
| |
* | More of jgross admits, less neg and the cmovsGravatar Rob Sloan2016-11-01
| |
* | most of jgross' admitsGravatar Rob Sloan2016-10-31
|/ | | | '
* Some work on proofs in src/Reflection/Z/Interpretations.vGravatar Jason Gross2016-10-27
|
* Add some rewrites and admitted lemmasGravatar Jason Gross2016-10-27
|
* Add beginnings of various interpretations of expression treesGravatar Jason Gross2016-10-27
|
* More 8.4 fixesGravatar Jason Gross2016-10-23
|
* Prove more things in WordUtilGravatar Jason Gross2016-10-23
| | | | The proofs should be automated eventually...
* Fill in some word util admitted lemmasGravatar Jason Gross2016-10-23
|
* Add word64eqb_ZeqbGravatar Jason Gross2016-10-21
|
* integrate bitwise operationsGravatar Andres Erbsen2016-10-12
|
* Generalize and simplify cast_word_reflGravatar Jason Gross2016-10-12
|
* word manipulation functions for secret key formatting (#74)Gravatar Andres Erbsen2016-10-12
| | | | | | | | | | * wordsize automation hooks and examples * wordToNat_cast_word * WordUtil: make [wordsize_eq] transparent * address code review comments
* Derive EdDSA.verify from equational specificationGravatar Andres Erbsen2016-09-16
| | | | Experiments/SpecEd25519 will come back soon
* Proved decode_point_eq in Ed25519 (comparing encodings is equivalent toGravatar jadep2016-04-29
| | | | comparing points).
* Cleanup: mostly moving lemmas to Util files, some moving lemmas to more ↵Gravatar jadep2016-04-28
| | | | general contexts.
* Finish absolutizing importsGravatar Jason Gross2016-03-10
| | | | | | | | | | | | The file coqprime/Coqprime/ListAux.v was importing List, which was confusing machines on which mathclasses was also installed. Using https://github.com/JasonGross/coq-tools ```bash make -kj10 cd src git ls-files "*.v" | xargs python ~/Documents/repos/coq-tools/absolutize-imports.py -i -R . Crypto ```
* Factor out some bedrock dependencies into WordUtilGravatar Jason Gross2016-02-25
Also move a definition about words, with a TODO about location, into WordUtil.