aboutsummaryrefslogtreecommitdiff
path: root/theories/Strings/HexString.v
AgeCommit message (Collapse)Author
2020-03-18Update headers in the whole code base.Théo Zimmermann
Add headers to a few files which were missing them.
2019-06-17Update headers of files that were stuck on older headers.Théo Zimmermann
Most of these files were introduced after #6543 but used older headers copied from somewhere else.
2018-12-12Avoid Fixpoint without struct nor body in stdlibMaxime Dénès
As reported in #9060, the STM does not handle such constructions properly. They are anyway fragile, for example Guarded reports a failure if run at the end of the scripts, so this patch is an improvement.
2018-07-16bin,oct,hex conversions positive,Z,N,nat<->stringJason Gross