aboutsummaryrefslogtreecommitdiff
path: root/theories/Strings
AgeCommit message (Expand)Author
2020-11-09Merge PR #13173: Lint stdlib with -mangle-names #4coqbot-app[bot]
2020-10-11Modify Strings/String.v to compile with -mangle-namesJasper Hugunin
2020-10-11Modify Strings/Ascii.v to compile with -mangle-namesJasper Hugunin
2020-10-05Adapting theories to unused pattern-matching variable warning.Hugo Herbelin
2020-03-18Update headers in the whole code base.Théo Zimmermann
2020-01-08Avoid hardcoded paths in extractionMaxime Dénès
2019-06-17Update headers of files that were stuck on older headers.Théo Zimmermann
2019-06-17Update ml-style headers to new year.Théo Zimmermann
2019-05-25Modifying theories to preferably use the "[= ]" syntax, and,Hugo Herbelin
2018-12-12Merge PR #9087: Add CI job building stdlib with `async-proofs on`Emilio Jesus Gallego Arias
2018-12-12Avoid Fixpoint without struct nor body in stdlibMaxime Dénès
2018-11-28Byte.v: use right-associative tuples in bitsJason Gross
2018-11-28Proofs to ensure that conversions round-tripJason Gross
2018-11-28Speed up ByteJason Gross
2018-11-28Add `String Notation` vernacular like `Numeral Notation`Jason Gross
2018-11-11Merge PR #8795: Encapsulating declarations of primitive string syntax in a mo...Jason Gross
2018-10-29NArith: add lemmas about numbers and vectorsYishuai Li
2018-10-23Encapsulating declarations of primitive string syntax in a module.Hugo Herbelin
2018-10-17Strings: add ByteVectorYishuai Li
2018-10-10[coqlib] Rebindable Coqlib namespace.Emilio Jesus Gallego Arias
2018-09-10Declaring Scope prior to loading primitive printers.Hugo Herbelin
2018-07-25Merge PR #8063: Direct implementation of Ascii.eqb and String.eqb (take 2)Hugo Herbelin
2018-07-16Add additional lemmas about {String,Ascii}.eqbJason Gross
2018-07-16Ascii.eqb and String.eqbPierre Letouzey
2018-07-16bin,oct,hex conversions positive,Z,N,nat<->stringJason Gross
2018-03-07Merge PR #6744: Add String.concatMaxime Dénès
2018-02-27Update headers following #6543.Théo Zimmermann
2018-02-24Add String.concatJason Gross
2017-07-04Bump year in headers.Pierre-Marie Pédrot
2017-06-01drop vo.itarget files and compute the corresponding the corresponding values ...Matej Kosik
2016-11-24Fix some documentation typos.Guillaume Melquiond
2016-06-18Giving a more natural semantics to injection by default.Hugo Herbelin
2016-01-20Update copyright headers.Maxime Dénès
2015-01-12Update headers.Maxime Dénès
2014-09-17Add some missing Proof statements.Guillaume Melquiond
2014-07-09Arith: full integration of the "Numbers" modular frameworkPierre Letouzey
2012-08-08Updating headers.herbelin
2012-07-05Kills the useless tactic annotations "in |- *"letouzey
2012-07-05Open Local Scope ---> Local Open Scope, same with Notation and aliiletouzey
2012-07-05ZArith + other : favor the use of modern names instead of compat notationsletouzey
2011-10-22Fixing Equality.injectable which did not detect an equality withoutherbelin
2010-07-24Updated all headers for 8.3 and trunkherbelin
2010-06-04Ascii: simplier ascii_of_pos, conversion from/to N, proofs about nat-->ascii-...letouzey
2010-04-29Remove the svn-specific $Id$ annotationsletouzey
2009-12-09Factorisation between Makefile and ocamlbuild systems : .vo to compile are in...letouzey
2009-11-02Remove various useless {struct} annotationsletouzey
2009-09-28Fix the stdlib doc compilation + switch all .v file to utf8letouzey
2009-09-17Delete trailing whitespaces in all *.{v,ml*} filesglondu
2009-03-27Parsing files for numerals (+ ascii/string) moved into pluginsletouzey
2008-06-20typo in a commentletouzey