| Age | Commit message (Collapse) | Author | |
|---|---|---|---|
| 2020-11-05 | Merge PR #12218: Numeral notations for non inductive types | coqbot-app[bot] | |
| Reviewed-by: herbelin Reviewed-by: JasonGross Reviewed-by: jfehrle Ack-by: Zimmi48 | |||
| 2020-11-02 | Merge PR #13247: Fixes #13241: nested Ltac functions wrongly reporting error ↵ | Pierre-Marie Pédrot | |
| on the inner calls Reviewed-by: ppedrot | |||
| 2020-10-30 | Renaming Numeral into Number | Pierre Roux | |
| 2020-10-29 | Fixing interpretation of rewrite_strat argument in Ltac. | Hugo Herbelin | |
| Ltac variables were not yet supported. | |||
| 2020-10-29 | Use same code for "Print Ltac foo" and "Print foo" when "foo" is an Ltac. | Hugo Herbelin | |
| Adopting the same format means printing "Ltac foo := ..." and not the fully qualified name of foo. | |||
| 2020-10-28 | Fixes #13241 (nested Ltac functions were wrongly reporting error on the ↵ | Hugo Herbelin | |
| inner calls). This continues #12223, #12773, #12992, #12774, #12999. | |||
| 2020-10-27 | Merge PR #13238: Fix some tactic print bugs | coqbot-app[bot] | |
| Reviewed-by: gares Reviewed-by: herbelin Ack-by: ppedrot | |||
| 2020-10-27 | Rename misc nonterminals | Jim Fehrle | |
| 2020-10-27 | Rename tactic_expr -> ltac_expr | Jim Fehrle | |
| 2020-10-27 | Rename operconstr -> term | Jim Fehrle | |
| 2020-10-27 | Merge PR #13075: Introducing the foundations for a name-alias-agnostic API | coqbot-app[bot] | |
| Reviewed-by: SkySkimmer Ack-by: gares Ack-by: ejgallego | |||
| 2020-10-26 | Improve tactic interpreter registration API a bit | Gaëtan Gilbert | |
| Using it feels nicer this way, with GADT details hidden inside comtactic | |||
| 2020-10-26 | Merge PR #13137: [ltac] Avoid magic numbers | coqbot-app[bot] | |
| Reviewed-by: herbelin | |||
| 2020-10-22 | Fix printing of wit_constr and some ssr problems with printing empty lists | Lasse Blaauwbroek | |
| 2020-10-22 | Make sure that setoid_rewrite passes state to subgoals | Lasse Blaauwbroek | |
| 2020-10-22 | Merge PR #13130: setoid_rewrite: record generated name when rewriting under ↵ | Pierre-Marie Pédrot | |
| lambda Reviewed-by: ppedrot | |||
| 2020-10-21 | Deprecate the non-qualified equality functions on kerpairs. | Pierre-Marie Pédrot | |
| This allows to quickly spot the parts of the code that rely on the canonical ordering. When possible we directly introduce the quotient-aware versions. | |||
| 2020-10-19 | Merge PR #13208: Support "Solve Obligations of <ident>" | coqbot-app[bot] | |
| Reviewed-by: SkySkimmer | |||
| 2020-10-19 | Merge PR #13197: Require at least one reference for Typeclasses ↵ | coqbot-app[bot] | |
| Opaque/Transparent Reviewed-by: SkySkimmer | |||
| 2020-10-16 | Merge PR #13195: Add support for "typeclasses eauto bfs <int_or_var_opt>" | Pierre-Marie Pédrot | |
| Reviewed-by: ppedrot | |||
| 2020-10-16 | Merge PR #13196: For "Typeclasses eauto", search depth should be a natural, ↵ | Pierre-Marie Pédrot | |
| not an integer Reviewed-by: ppedrot | |||
| 2020-10-15 | Support "Solve Obligations of <ident>" option | Jim Fehrle | |
| 2020-10-15 | Require at least one reference for Typeclasses Opaque/Transparent | Jim Fehrle | |
| (zero references is currently a no-op) | |||
| 2020-10-14 | For "Typeclasses eauto", search depth should be a natural, not an | Jim Fehrle | |
| integer | |||
| 2020-10-14 | Add support for "typeclasses eauto bfs <int_or_var_opt> | Jim Fehrle | |
| 2020-10-14 | Deprecating wit_var to the benefit of its synonymous wit_hyp. | Hugo Herbelin | |
| Note: "hyp" was documented in Ltac Notation chapter but "var" was not. | |||
| 2020-10-10 | Prim.pattern_ident takes a location and its synonymous pattern_identref is ↵ | Hugo Herbelin | |
| deprecated. | |||
| 2020-10-09 | Merge PR #13088: [stm] move par: to comTactic | coqbot-app[bot] | |
| Reviewed-by: SkySkimmer Reviewed-by: ppedrot Reviewed-by: ejgallego | |||
| 2020-10-09 | [stm] move par: implementation to vernac/comTactic and stm/partac | Enrico Tassi | |
| The current implementation of par: is still in the STM, but is optional. If the STM does not take over it, it defaults to the implementation of in comTactic which is based on all: (i.e. sequential). This commit also moved the interpretation of a tactic from g_ltac to vernac/comTactic which is more appropriate. Co-authored-by: Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net> | |||
| 2020-10-08 | Dropping the misleading int argument of Pp.h. | Hugo Herbelin | |
| An h-box inhibits the breaking semantics of any cut/spc/brk in the enclosed box. We tentatively replace its occurrence by an h or hv, assuming in particular that if the indentation is not 0, an hv box was intended. | |||
| 2020-10-07 | Merge PR #13115: Derive Inversion does not allow leftover evars | Pierre-Marie Pédrot | |
| Reviewed-by: ppedrot | |||
| 2020-10-07 | Merge PR #13119: Fix retyping anomaly in rewrite | Pierre-Marie Pédrot | |
| Reviewed-by: ppedrot | |||
| 2020-10-04 | Merge PR #13096: Drop prefixes from non-terminal names, e.g. "constr:constr" ↵ | coqbot-app[bot] | |
| -> "constr" Reviewed-by: herbelin Ack-by: Zimmi48 | |||
| 2020-10-04 | Remove prefixes on nonterminal names, e.g. "constr:" and "Prim." | Jim Fehrle | |
| 2020-10-03 | Avoid magic numbers | Jim Fehrle | |
| 2020-10-02 | setoid_rewrite: record generated name when rewriting under lambda | Gaëtan Gilbert | |
| Fix #13129 | |||
| 2020-10-02 | Cleanup rewrite.ml | Gaëtan Gilbert | |
| Remove unused arguments and commented code | |||
| 2020-09-30 | Fix retyping anomaly in rewrite | Gaëtan Gilbert | |
| Fix #13045 Also make sure future anomalies won't be fed to tclzero. Instead of retyping with lax:true we may question why we produce an ill-typed term in decompose_app_rel: in the | App (f, [|arg|]) -> case we produce `fun x y : T => bla x y` but we have no assurance that the second argument of `bla` should have type `T`. | |||
| 2020-09-30 | Further simplification of the typeclass registration API. | Pierre-Marie Pédrot | |
| 2020-09-30 | Derive Inversion does not allow leftover evars | Gaëtan Gilbert | |
| Fix #12917 | |||
| 2020-09-25 | Merge PR #12999: More improvements in locating tactic errors | coqbot-app[bot] | |
| Reviewed-by: ppedrot Reviewed-by: ejgallego | |||
| 2020-09-22 | Fixes #9716, #13004: don't drop the qualifier of quotations at printing time. | Hugo Herbelin | |
| 2020-09-18 | Merge PR #12963: Formally deprecate the double induction tactic. | Hugo Herbelin | |
| Reviewed-by: VincentSe Ack-by: herbelin Ack-by: olaure01 | |||
| 2020-09-17 | [leminv] Use higher-level Declare API. | Emilio Jesus Gallego Arias | |
| 2020-09-17 | [leminv] Remove unused catch. | Emilio Jesus Gallego Arias | |
| 2020-09-17 | Formally deprecate the double induction tactic. | Pierre-Marie Pédrot | |
| The doc states it is deprecated since 1386cd9 but this was ages before the deprecation mechanism existed. | |||
| 2020-09-16 | More improvements in locating tactic errors. | Hugo Herbelin | |
| We finally pass the location in the "ist", and keep it in the "VFun" which is associated to expanded Ltac constants. | |||
| 2020-09-11 | Adding a wit_natural standard argument. | Hugo Herbelin | |
| 2020-09-11 | Turn integer into natural in several mlgs | Pierre Roux | |
| Negative values had no meaning there. Those were spotted by Hugo Herbelin while reviewing #12979 . | |||
| 2020-09-11 | [refman] Rename int to integer | Pierre Roux | |
