aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Making parentheses mandatory in tactic scopes.Gravatar Pierre-Marie Pédrot2016-03-04
|
* Uniformizing the parsing of argument scopes in Ltac.Gravatar Pierre-Marie Pédrot2016-03-04
|
* Merge pull request #97 from clarus/trunkGravatar Pierre-Marie Pédrot2016-03-04
|\ | | | | Converting the README to MarkDown syntax.
* \ Merge branch 'clean-atomic-tactics'Gravatar Pierre-Marie Pédrot2016-02-29
|\ \
| * | Moving the "move" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
| | |
| * | Moving the "exists" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
| | |
| * | Moving the "symmetry" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
| | |
| * | Moving the "generalize dependent" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
| | |
| * | Moving the "clearbody" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
| | |
| * | Moving the "clear" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
| | |
| * | Moving the "cofix" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
| | |
| * | Moving the "fix" tactic to TACTIC EXTEND.Gravatar Pierre-Marie Pédrot2016-02-29
|/ /
* | Printing notations: Cleaning in anticipation of fixing #4592.Gravatar Hugo Herbelin2016-02-28
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | - Making a clear distinction between expressions of the notation which are associated to binding variables only (as in `Notation "'lam' x , P" := (fun x => P)" or `Notation "'exists2' x : t , p & q" := (ex2 (fun x:t => p) (fun x:t => q))') and those which are associated to at list one subterm (e.g. `Notation "x .+1" := (S x)' but also "Notation "{# x | P }" := (ex2 _ (fun y => x = F y) (fun x => P))' as in #4592). The former have type NtnTypeOnlyBinder. - Thus avoiding in particular encoding too early Anonymous as GHole and "Name id" as "GVar id". There is a non-trivial alpha-conversion work to do to get #4592 working. See comments in Notation_ops.add_env.
* | Slightly contracting code of evarconv.ml.Gravatar Hugo Herbelin2016-02-28
| |
* | Removing Tacmach.New qualification in Tacinterp.Gravatar Pierre-Marie Pédrot2016-02-27
| |
* | Removing some compatibility layers in Tacinterp.Gravatar Pierre-Marie Pédrot2016-02-27
| |
* | Qcabs : absolute value on normalized rational numbers QcGravatar Pierre Letouzey2016-02-26
| | | | | | | | | | | | | | | | File contributed by Cédric Auger (a long time ago, sorry!) Qarith and Qc would probably deserve many more results like this one, and a more modern style (for instance qualified names), but this commit is better than nothing...
* | Qcanon : fix names of lemmas Qcle_alt & Qcge_alt (were Qle_alt & Qge_alt)Gravatar Pierre Letouzey2016-02-26
| |
* | Qcanon : implement some old suggestions by C. AugerGravatar Pierre Letouzey2016-02-26
| |
* | Merge branch 'remove-quotations'Gravatar Pierre-Marie Pédrot2016-02-24
|\ \
| * | Removing the METAIDENT token, as it is not used anymore.Gravatar Pierre-Marie Pédrot2016-02-24
| | | | | | | | | | | | | | | | | | METAIDENT were idents of the form $foobar, only used in quotations. Note that it removes two dollars in the Coq codebase! Guess I'm absolved for the $(...) syntax.
| * | Removing the MetaIdArg entry of tactic expressions.Gravatar Pierre-Marie Pédrot2016-02-24
| | | | | | | | | | | | | | | | | | This was historically used together with the <:tactic< ... >> quotation to insert foreign code as $foo, but it actually only survived in the implementation of Tauto. With the removal of the quotation feature, this is now totally obsolete.
| * | Removing the Q_coqast module.Gravatar Pierre-Marie Pédrot2016-02-24
| | | | | | | | | | | | | | | | | | It implemented the quotation logic of terms and tactics, although it was mostly obsolete. With quotations gone, it is now useless and thus removed. I fundamentally doubt that anyone hardly depends on this out there.
| * | Getting rid of the "<:tactic< ... >>" quotations.Gravatar Pierre-Marie Pédrot2016-02-24
|/ / | | | | | | | | | | | | It used to allow to represent parts of tactic AST directly in ML code. Most of the uses were trivial, only calling a constant, except for tauto that had an important code base written in this style. Removing this reduces the dependency to CAMLPX and the preeminence of Ltac in ML code.
* | Moving tauto.ml4 to a proper ML file.Gravatar Pierre-Marie Pédrot2016-02-23
| |
* | Moving the Tauto tactic to proper Ltac.Gravatar Pierre-Marie Pédrot2016-02-22
| | | | | | | | | | | | This gets rid of brittle code written in ML files through Ltac quotations, and reduces the dependance of Coq to such a feature. This also fixes the particular instance of bug #2800, although the underlying issue is still there.
* | The tactic generic argument now returns a value rather than a glob_expr.Gravatar Pierre-Marie Pédrot2016-02-22
| | | | | | | | | | | | | | | | | | | | The glob_expr was actually always embedded as a VFun, so this patch should not change anything semantically. The only change occurs in the plugin API where one should use the Tacinterp.tactic_of_value function instead of Tacinterp.eval_tactic. Moreover, this patch allows to use tactics returning arguments from the ML side.
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-02-21
|\ \
| * | Fixing bug #4540: CoqIDE bottom progress bar does not update.Gravatar Pierre-Marie Pédrot2016-02-20
| | |
| * | Fix regression from 8.4 in reflexivity/...Gravatar Matthieu Sozeau2016-02-19
| | | | | | | | | | | | | | | reflexivity/symmetry/transitivity only need RelationClasses to be loaded.
* | | Merge branch 'located-universes'Gravatar Pierre-Marie Pédrot2016-02-19
|\ \ \
| * | | Adding location to universes generated by the pretyper.Gravatar Pierre-Marie Pédrot2016-02-19
| | | |
| * | | Allowing to attach location to universes in UState.Gravatar Pierre-Marie Pédrot2016-02-19
|/ / /
| * | Fixing bug #4580: [Set Refine Instance Mode] also used for Program Instance.Gravatar Pierre-Marie Pédrot2016-02-19
| | |
| * | Fixing bug #4582: cannot override notation [ x ].Gravatar Pierre-Marie Pédrot2016-02-19
| | |
| * | STM: Print/Extraction have to be skipped if -quickGravatar Enrico Tassi2016-02-19
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Print and Extraction commands may pierce opacity: if the task producing the proof term is not finished, we wait for its completion. In -quick mode no worker is going to process a task, since tasks are simply stored to disk (and resumed later in -vio2vo mode). This commit avoids coqc waits forever for a task in order to Print/Extract the corresponding term. Bug reported privately by Alec Faithfull.
| * | CoqIDE: STOP button also stops workers (fix #4542)Gravatar Enrico Tassi2016-02-19
| | |
| * | STM: classify some variants of Instance as regular `Fork nodes.Gravatar Enrico Tassi2016-02-19
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | "Instance name : Type." is like "Lemma name : Type", i.e. it starts a proof. Unfortunately sometimes it does not, so we say VtUnknown. Still, if there is an open proof, we classify it as a regular Lemma, i.e. the opacity depends only on the terminator. This makes CoqIDE and PIDE based UI way more responsive when processing files containing Instance that are proved by tactics, since they are now correctly delegated to workers. Bug reported privately by Alec Faithfull.
* | | FIX: of my previous merging mistakeGravatar Matej Kosik2016-02-18
| | |
* | | ADD: Names.Name.is_{anonymous,name}Gravatar Matej Kosik2016-02-18
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Two new (trivial) functions were added: Names.Name.is_anonymous : Names.Name.t -> bool Names.Name.is_name : Names.Name.t -> bool They enable us to write a more compact code. (example: commit "99633f4" in "relation-extraction" module of "coq-contribs").
| * | Fixing the Proofview.Goal.goal function.Gravatar Pierre-Marie Pédrot2016-02-17
| | | | | | | | | | | | | | | The environment put in the goals was not the right one and could lead to various leaks.
| * | Fix bug #4574: Anomaly: Uncaught exception Invalid_argument("splay_arity").Gravatar Pierre-Marie Pédrot2016-02-17
| | | | | | | | | | | | | | | The setoid_rewrite tactic was not checking that the relation it was looking for was indeed a relation, i.e. that its type was an arity.
* | | CLEANUP: Context.{Rel,Named}.Declaration.tGravatar Matej Kosik2016-02-17
|\ \ \
* | | | CLEANUP: Renaming "Util.compose" function to "%"Gravatar Matej Kosik2016-02-17
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | I propose to change the name of the "Util.compose" function to "%". Reasons: 1. If one wants to express function composition, then the new name enables us to achieve this goal easier. 2. In "Batteries Included" they had made the same choice.
* | | | Tacticals: typo in a commentGravatar Pierre Letouzey2016-02-16
| | | |
* | | | Term: fix a comment (first de Bruijn index is 1)Gravatar Pierre Letouzey2016-02-16
| | | |
| * | | Renaming variants of Entries.local_entryGravatar Matej Kosik2016-02-16
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | The original datatype: Entries.local_entry = LocalDef of constr | LocalAssum of constr was changed to: Entries.local_entry = LocalDefEntry of constr | LocalAssumEntry of constr There are two advantages: 1. the new names are consistent with other variant names in the same module which also have this "*Entry" suffix 2. the new names do not collide with variants defined in the Context.{Rel,Named}.Declaration modules so both, "Entries" as well as "Context.{Rel,Named}.Declaration" can be open at the same time. The disadvantage is that those new variants are longer. But since those variants are rarely used, it it is not a big deal.
| * | | CLEANUP: Simplifying the changes done in "checker/*"Gravatar Matej Kosik2016-02-15
| | | |
| * | | merging conflicts with the original "trunk__CLEANUP__Context__2" branchGravatar Matej Kosik2016-02-15
|/| | |
* | | | Using monotonic types for conversion functions.Gravatar Pierre-Marie Pédrot2016-02-15
| | | |