index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
test-suite
/
success
/
ProgramWf.v
Age
Commit message (
Expand
)
Author
2021-04-02
Remove the omega tactic and related options
Jim Fehrle
2019-04-16
Fix spurious argument of {measure}
Maxime Dénès
2019-04-16
Take advantage of relaxed {measure} syntax in test suite
Maxime Dénès
2017-08-21
Ensuring all .v files end with a newline to make "sed -i" work better on them.
Hugo Herbelin
2012-07-05
Open Local Scope ---> Local Open Scope, same with Notation and alii
letouzey
2012-07-05
ZArith + other : favor the use of modern names instead of compat notations
letouzey
2012-03-19
Fix bugs related to Program integration.
msozeau
2011-11-30
Quick hack to avoid anomaly on using Program w/o having required JMeq.
herbelin
2009-11-13
Fix test-suite scripts: [Generalizable Variables] and small
msozeau
2009-09-22
Add the option to automatically introduce variables declared before the
msozeau
2009-09-17
Delete trailing whitespaces in all *.{v,ml*} files
glondu
2009-03-29
Avoid inadvertent declaration of "on" as a keyword. New syntax is
msozeau
2009-03-28
Rewrite of Program Fixpoint to overcome the previous limitations:
msozeau