index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
tactics
Age
Commit message (
Expand
)
Author
2019-12-11
Merge PR #11271: Fixing #9893. "Specialize with" would not support hyps type ...
Pierre-Marie Pédrot
2019-12-10
Fixing #9893 (Letins not supported in the specialized hypothesis).
Pierre Courtieu
2019-12-10
Side-effect free wrapper around already declared schemes.
Pierre-Marie Pédrot
2019-12-10
Make explicit that users should not observe return values of scheme functions.
Pierre-Marie Pédrot
2019-12-10
Simplify internal flags in scheme declarations.
Pierre-Marie Pédrot
2019-12-06
Moving the diversity of constr printers to a label style.
Hugo Herbelin
2019-11-30
Actually deprecate the `cutrewrite` tactic
Maxime Dénès
2019-11-21
[coq] Untabify the whole ML codebase.
Emilio Jesus Gallego Arias
2019-11-11
Do not export the internals of the prepare_hint function.
Pierre-Marie Pédrot
2019-11-08
Make [Proof_global.closed_proof_output] opaque
Gaëtan Gilbert
2019-11-01
Add primitive float computation in Coq kernel
Guillaume Bertholon
2019-10-30
[declare] Remove declare_scheme hook in Declare
Emilio Jesus Gallego Arias
2019-10-30
Merge PR #10981: [abstract] Remove un-unused reference to `evar_map`
Pierre-Marie Pédrot
2019-10-30
Merge PR #10949: [declare] Provide helper for private constant inlining.
Pierre-Marie Pédrot
2019-10-30
Merge PR #10681: [declare] Make `proof_entry` a private type.
Pierre-Marie Pédrot
2019-10-30
Merge PR #10494: Show diffs in "Show Proof."
Enrico Tassi
2019-10-29
Show diffs in "Show Proof."
Jim Fehrle
2019-10-29
[abstract] Remove un-unused reference to `evar_map`
Emilio Jesus Gallego Arias
2019-10-29
[declare] Use helper function for `fix_exn` instead of relying on internals.
Emilio Jesus Gallego Arias
2019-10-29
[declare] Make `proof_entry` a private type.
Emilio Jesus Gallego Arias
2019-10-28
[declare] Provide helper for private constant inlining.
Emilio Jesus Gallego Arias
2019-10-24
[declare] Split inductive declaration code to vernac/
Emilio Jesus Gallego Arias
2019-10-24
[declare] Split universe declaration code to vernac/
Emilio Jesus Gallego Arias
2019-10-16
Simplify future forcing in Declare.
Pierre-Marie Pédrot
2019-10-16
Ensure that side-effect declarations reaching the kernel are forced.
Pierre-Marie Pédrot
2019-10-16
Split the function used to declare side-effects from the standard one.
Pierre-Marie Pédrot
2019-10-16
Cleaning up the previous code by ensuring statically invariants on opaque pro...
Pierre-Marie Pédrot
2019-10-14
Use kernel info from Global for Lib.sections_{depth,are_opened}
Gaëtan Gilbert
2019-10-14
Remove [in_section] arguments to Safe_typing functions
Gaëtan Gilbert
2019-10-13
Merge PR #10862: Simplify universe handling wrt side effects: rm demote_seff_...
Pierre-Marie Pédrot
2019-10-13
Merge PR #10670: ComAssumption cleanup
Pierre-Marie Pédrot
2019-10-11
Merge PR #10804: Fix Print All of section variables
Pierre-Marie Pédrot
2019-10-09
Specialize UState.merge for extend:false
Gaëtan Gilbert
2019-10-09
Simplify universe handling wrt side effects: rm demote_seff_univs
Gaëtan Gilbert
2019-10-05
Remove "is_polymorphic_univ" checks in upper layers.
Gaëtan Gilbert
2019-10-05
Declare universes for variables outside of Declare.declare_variable
Gaëtan Gilbert
2019-10-04
Remove redundancy in section hypotheses of kernel entries.
Pierre-Marie Pédrot
2019-10-01
Fix Print All of section variables
Gaëtan Gilbert
2019-09-28
Remove the monomorphic universe libobject.
Pierre-Marie Pédrot
2019-09-26
Implement section discharging inside kernel.
Pierre-Marie Pédrot
2019-09-25
Move the Lib section data into the kernel.
Pierre-Marie Pédrot
2019-09-25
Refine the API to declare section-local universes.
Pierre-Marie Pédrot
2019-09-04
Merge PR #10612: Fix feedback levels
Emilio Jesus Gallego Arias
2019-08-30
Merge PR #10714: Solve universe error with SSR 'rewrite !term'
Pierre-Marie Pédrot
2019-08-29
Solve universe error with SSR 'rewrite !term'
Andreas Lynge
2019-08-29
Merge PR #10674: [declare] Move proof_entry type to declare, put interactive ...
Pierre-Marie Pédrot
2019-08-29
Merge PR #10660: [cleanup] Replace uses of UserError constructor, clarify exc...
Pierre-Marie Pédrot
2019-08-29
Make sure that all query commands return a notice (not an info) feedback
Maxime Dénès
2019-08-27
[declare] Use entry constructor instead of low-level record.
Emilio Jesus Gallego Arias
2019-08-27
[declare] Move proof_entry type to declare, put interactive proof data on top...
Emilio Jesus Gallego Arias
[next]