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.
reactivate Thm.check_hyps, after adapting AFP/Datatype_Order_Generator (see AFP/b7e389b5765c);
2014-01-11, by wenzelm
check_hyps for attribute application (still inactive, due to non-compliant tools);
2014-01-11, by wenzelm
clarified context;
2014-01-11, by wenzelm
clarified context;
2014-01-11, by wenzelm
tuned signature;
2014-01-11, by wenzelm
shot in the dark to make LaTeX happy again
2014-01-11, by haftmann
provide default name in splitted representation
2014-01-11, by haftmann
dropped legacy alias feature
2014-01-11, by haftmann
merged
2014-01-10, by wenzelm
disable Thm.check_hyps for now, due to remaining problems with AFP/Datatype_Order_Generator and AFP/Psi_Calculi (because of HOL-Nominal 'equivariance');
2014-01-10, by wenzelm
more elementary management of declared hyps, below structure Assumption;
2014-01-10, by wenzelm
more accurate context;
2014-01-10, by wenzelm
tuned;
2014-01-10, by wenzelm
explicit check of background theory;
2014-01-10, by wenzelm
basic ordinal arithmetic and cardinals library extension (not relevant for BNFs)
2014-01-10, by traytel
correctly extract code RHS, with loose bound variables
2014-01-10, by blanchet
cope gracefully with missing ctr equations by plugging in 'False ==> ...'
2014-01-10, by blanchet
strengthened tactic to handle 'disc_iff' equations of the form '... = False'
2014-01-10, by blanchet
repair 'exhaustive' feature for one-constructor types
2014-01-10, by blanchet
pass right rhs as code rhs
2014-01-10, by blanchet
use correct default for exclude rules to avoid weird tactic failures
2014-01-10, by blanchet
tuning (no need for |-> here)
2014-01-10, by blanchet
fix 'primcorec' (as opposed to 'primcorecursive') with 'exhaustive')
2014-01-10, by blanchet
tuning
2014-01-10, by blanchet
only destruct cases equipped with the right stuff (in particular, 'sel_split')
2014-01-10, by blanchet
generate 'disc_iff' for all discriminators
2014-01-10, by blanchet
use 'disc_iff' as simp rules whenever possible + clean up '= True', '= False', etc.
2014-01-10, by blanchet
exhaustive rules like '(False ==> P) ==> P ==> P' are now filtered out as trivial
2014-01-10, by blanchet
merged
2014-01-10, by wenzelm
more robust;
2014-01-10, by wenzelm
merged
2014-01-10, by wenzelm
tuned;
2014-01-09, by wenzelm
access X11 window manager;
2014-01-09, by wenzelm
new codatatype example: stream processors
2014-01-10, by traytel
use the right context in tactic
2014-01-10, by traytel
fixed 'disc_iff' tactic in the case where different equations use different variable names for the function arguments
2014-01-10, by blanchet
do not use wrong constructor in auto-generated proof goal
2014-01-09, by panny
fixed de Bruijn bug in 'unfold_lets'
2014-01-09, by blanchet
tuned error message
2014-01-09, by blanchet
reintroduce recursive calls under constructors, taken out in 8dd0e0316881 mainly and in subsequent changes
2014-01-09, by blanchet
strengthened tactics w.r.t. 'lets' and tuples
2014-01-09, by blanchet
strengthen tac w.r.t. lets with tuples
2014-01-09, by blanchet
use 'prove_sorry'
2014-01-09, by blanchet
for code equations that coincide with ctr equations, make sure the usr's input is preserved for both
2014-01-09, by blanchet
made 'datatype_new_compat' work with sort constraints
2014-01-09, by blanchet
merge
2014-01-08, by panny
match order of generated theorems to user input;
2014-01-08, by panny
typo
2014-01-08, by kuncar
ensure that schematic type variables are fresh in rty
2014-01-08, by kuncar
ensure that the raw type of an abstract type cannot be treated as an abstract type recursively
2014-01-08, by kuncar
tuned
2014-01-08, by nipkow
avoid hard tabs in output -- somewhat ill-defined;
2014-01-07, by wenzelm
uniform output of tracing via official channel (usually depending on trace flag);
2014-01-07, by wenzelm
tuned
2014-01-07, by nipkow
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip