Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
merged
2014-01-06, by wenzelm
more informative error message;
2014-01-06, by wenzelm
obsolete / unmaintained;
2014-01-06, by wenzelm
misc tuning and clarification;
2014-01-06, by wenzelm
more formal ISABELLE_BROWSER_INFO;
2014-01-06, by wenzelm
tuned comments;
2014-01-06, by wenzelm
dropped legacy
2014-01-06, by haftmann
order and graph for code symbols
2014-01-06, by haftmann
special treatment of ==> and == solely as constants
2014-01-06, by haftmann
uniform orientation of instances as (type constructor, type class)
2014-01-06, by haftmann
minimized class dependency, updated references
2014-01-05, by nipkow
proper context for simplifier invocations in code generation stack
2014-01-03, by haftmann
spelling
2014-01-03, by haftmann
proper name generation to avoid clash with 'P' in user specification
2014-01-03, by blanchet
more SML-ish (less Haskell-ish) naming convention
2014-01-03, by blanchet
strengthened tactic
2014-01-03, by blanchet
refactoring
2014-01-03, by blanchet
instantiate schematics as projections to avoid HOU trouble
2014-01-03, by blanchet
tuning
2014-01-03, by blanchet
avoid schematic variable in goal, which sometimes gets instantiated by tactic
2014-01-02, by blanchet
generalized tactic to the case of several assumptions per equation
2014-01-02, by blanchet
made tactic behave better w.r.t. HO unification (might not be enough, and might have to fix some variables eventually though...)
2014-01-02, by blanchet
made tactic more robust
2014-01-02, by blanchet
made tactic handle corner cases, where some of the 'disc' properties are missing, correctly
2014-01-02, by blanchet
simplified code
2014-01-02, by blanchet
prevent tactic from getting out of sync and wrongly attack next subgoal
2014-01-02, by blanchet
removed pointless warning (cf. http://stackoverflow.com/questions/20233463/isabelle-metis-proof-state-contains-the-universal-sort/20785045#20785045)
2014-01-02, by blanchet
consider code as exhaustive
2014-01-02, by blanchet
proper handling of corner case, take 2
2014-01-02, by blanchet
robustness
2014-01-02, by blanchet
properly synchronize parallel lists
2014-01-02, by blanchet
graceful handling of one-constructor case
2014-01-02, by blanchet
gracefully handle single-equation case, where 'nchotomy' is 'True'
2014-01-02, by blanchet
made tactic handle gracefully the case of missing constructors
2014-01-02, by blanchet
removed 'nchotomy' property
2014-01-02, by blanchet
don't generate any proof obligation for implicit (de facto) exclusiveness
2014-01-02, by blanchet
detect syntactic exhaustiveness
2014-01-02, by blanchet
internally allow different values for 'exhaustive' for different constructors
2014-01-02, by blanchet
internally allow different values for 'sequential' for different constructors
2014-01-02, by blanchet
use same name for feature internally as in user interface, to facilitate grepping
2014-01-02, by blanchet
generate 'disc_iff' property in 'primcorec'
2014-01-02, by blanchet
added tactic to prove 'disc_iff' properties in 'primcorec'
2014-01-02, by blanchet
merged
2014-01-01, by wenzelm
clarified blast after change of SELECT_GOAL in 210bca64b894: do not smash flex-flex pairs of overall goal state (in analogy to maxidx) -- NB: Isar goal structure serves as natural boundary, e.g. in "by blast";
2014-01-01, by wenzelm
updated keywords;
2014-01-01, by wenzelm
clarified simplifier context;
2014-01-01, by wenzelm
simplified settings for src/HOL/Tools/SMT;
2014-01-01, by wenzelm
avoid unicode text, which causes problems when recoding symbols (e.g. via UTF8-Isabelle in Isabelle/jEdit);
2014-01-01, by wenzelm
dropped obsolete references to recdef
2014-01-01, by haftmann
examples how to avoid the "code, code del" antipattern
2014-01-01, by haftmann
fundamental treatment of undefined vs. universally partial replaces code_abort
2014-01-01, by haftmann
explicit distinction between empty code equations and no code equations, including convenient declaration attributes
2014-01-01, by haftmann
tuned whitespace
2014-01-01, by haftmann
more precise wording
2014-01-01, by haftmann
uniform bookkeeping also in the case of deletion
2014-01-01, by haftmann
more abstract declaration of code attributes
2013-12-31, by haftmann
dropped unused material
2013-12-31, by haftmann
proper context for norm_hhf and derived operations;
2013-12-31, by wenzelm
made SML/NJ happy;
2013-12-31, by wenzelm
added system option "jedit_print_mode";
2013-12-30, by wenzelm
avoid hardwired /bin/bash (like canonical Isabelle shell scripts);
2013-12-30, by wenzelm
tuned whitespace;
2013-12-30, by wenzelm
simplified
2013-12-29, by haftmann
more compact representation of different situations for interpretation
2013-12-29, by haftmann
more succint formulation of special case
2013-12-29, by haftmann
tuned whitespace
2013-12-29, by haftmann
move instantiation here from AFP/Native_Word
2013-12-28, by haftmann
dropped junk
2013-12-28, by haftmann
postpone dis"useful" lemmas
2013-12-28, by haftmann
cleanup
2013-12-28, by haftmann
prefix disambiguation
2013-12-28, by haftmann
tuned proofs and declarations
2013-12-27, by haftmann
prefer target-style syntaxx for sublocale
2013-12-27, by haftmann
prefer ephemeral interpretation over interpretation in proof contexts;
2013-12-26, by haftmann
self-contained formulation of subclass command, avoiding hard-wired Named_Target.init
2013-12-25, by haftmann
ephemeral interpretation also formally works on theory level
2013-12-25, by haftmann
abolished slightly odd global lattice interpretation for min/max
2013-12-25, by haftmann
prefer more canonical names for lemmas on min/max
2013-12-25, by haftmann
explicit distributivity facts on min/max
2013-12-25, by haftmann
postponed min/max lemmas until abstract lattice is available
2013-12-25, by haftmann
tuned structure of min/max lemmas
2013-12-25, by haftmann
prefer abstract simp rule
2013-12-25, by haftmann
more lemmas on abstract lattices
2013-12-25, by haftmann
tuning and augmentation of min/max lemmas;
2013-12-24, by haftmann
more general induction rule;
2013-12-24, by haftmann
convenient printing of polynomial values
2013-12-23, by haftmann
prefer "Bits" as theory name for abstract bit operations, similar to "Orderings", "Lattices", "Groups" etc.
2013-12-23, by haftmann
prefer Y_of_X over X_to_Y;
2013-12-23, by haftmann
merge
2013-12-23, by panny
prevent ambiguity when mutual recursion maps a datatype to itself, which yielded wrong definitions in some cases (e.g. nat)
2013-12-23, by panny
NEWS
2013-12-23, by haftmann
dropped redundant lemma
2013-12-23, by haftmann
syntactically tuned
2013-12-23, by haftmann
prefer plain bool over dedicated type for binary digits
2013-12-23, by haftmann
tuned
2013-12-23, by nipkow
compile + reduce problem size by a notch
2013-12-21, by blanchet
generate exhaust from nchotomy
2013-12-21, by blanchet
made tactic work with theorems with multiple assumptions
2013-12-21, by blanchet
renamed 'exhaust' to 'nchotomy' since it's expressed in the object logic (cf. datatype package)
2013-12-21, by blanchet
express weak pullback property of bnfs only in terms of the relator
2013-12-18, by traytel
merged
2013-12-20, by nipkow
tuned
2013-12-20, by nipkow
reconstruct SPASS-Pirate steps of the form 'x ~= C x' (or more complicated)
2013-12-20, by blanchet
tuning whitespace
2013-12-20, by blanchet
recognize datatype reasoning in SPASS-Pirate
2013-12-20, by blanchet
note manually proved exclusiveness property
2013-12-20, by blanchet
note exhaust proof obligation
2013-12-20, by blanchet
compile
2013-12-20, by blanchet
implemented 'exhaustive' option in tactic
2013-12-19, by blanchet
tuning
2013-12-19, by blanchet
tuning
2013-12-19, by blanchet
tuning 'case' expressions
2013-12-19, by blanchet
don't do 'isar_try0' if preplaying is off
2013-12-19, by blanchet
more data structure refactoring
2013-12-19, by blanchet
data structure rationalization
2013-12-19, by blanchet
tuning
2013-12-19, by blanchet
refactored preplaying outcome data structure
2013-12-19, by blanchet
distinguish not preplayed & timed out
2013-12-19, by blanchet
pick up tfree/tvar type from SPASS-Pirate proof
2013-12-19, by blanchet
tuning
2013-12-19, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip