Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+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.
add congruence rule to prevent code_simp from looping
2013-10-09, by Andreas Lochbihler
Added tag Isabelle2013-1-RC2 for changeset 782e430e6a83
2013-10-09, by wenzelm
native executable for Linux (see Admin/Linux);
2013-10-07, by wenzelm
proper NULL termination;
2013-10-07, by wenzelm
native executable even for Linux, to avoid surprises with file managers opening executable script as text file;
2013-10-07, by wenzelm
proper warning at run time, not in the parser;
2013-10-07, by wenzelm
prefer "fresh" open -- requires Lion / Mountain Lion;
2013-10-07, by wenzelm
clarified remove_overlay: always flush in order to make sure that apply_query can make a fresh start with the same arguments (see also 6e69f9ca8f1c) -- NB: print functions are idempotent;
2013-10-07, by wenzelm
prevent explosion in monomorphizer (e.g. when the facts typerep_int_def typerep_num_def typerep_option_def typerep_node_def are selected)
2013-10-04, by blanchet
more parallelism in blocking mode
2013-10-04, by blanchet
count remote threads as well when balancing CPU usage -- otherwise jEdit users and other users of the "blocking" mode may have to wait for 2 * timeout if they e.g. have 4 cores and 5 provers (the typical situation)
2013-10-04, by blanchet
another shortcut alias;
2013-10-04, by wenzelm
NEWS;
2013-10-04, by wenzelm
Added tag Isabelle2013-1-RC1 for changeset c37100233af7
2013-10-03, by wenzelm
reintroduced check from bd36da55d825 after all, due to hard-to-solve issues outside the N2M code
2013-11-11, by blanchet
removed dead code
2013-11-11, by blanchet
added check to avoid odd situations the N2M code cannot handle
2013-11-11, by blanchet
reverted check introduced in ce58fb149ff6, now that independent functions are allowed (cf. 347c3b0cab44)
2013-11-11, by blanchet
tuned signature
2013-11-11, by blanchet
handle independent functions defined in parallel in N2M (in presence of type variables, see ce58fb149ff6)
2013-11-11, by traytel
tuned
2013-11-11, by nipkow
tuned
2013-11-11, by nipkow
qualifed popular user space names
2013-11-10, by haftmann
dropped obsolete check: dest_num always yields positive number
2013-11-10, by haftmann
simplified: negative number is trivially smaller than 2, and SMT_Builtin.is_builtin_num implies that its argument is a number
2013-11-10, by haftmann
more exercises
2013-11-08, by nipkow
by (auto ...)[1] not by (auto [1])
2013-11-08, by blanchet
added exercise
2013-11-08, by nipkow
Add output translation for <a := .., b := .., ..> state notation.
2013-11-07, by kleing
reintroduce mutually (co)rec check, since the underlying N2M code doesn't quite handle the general case (esp. in presence of type variables)
2013-11-07, by blanchet
more docs
2013-11-07, by blanchet
properly detect when to perform n2m -- e.g. handle the case of two independent functions on irrelevant types being defined in parallel
2013-11-07, by blanchet
reverted 3e1d230f1c00 -- pervasiveness is useful, cf. Coinductive_Nat in the AFP
2013-11-06, by blanchet
simplified code
2013-11-06, by blanchet
fourth attempt at generalizing N2M types (to leverage caching)
2013-11-06, by blanchet
tuning
2013-11-06, by blanchet
int and nat are conditionally_complete_lattices
2013-11-05, by hoelzl
be more open-minded and allow needless mutual recursion for 'prim(co)rec', since we allow it for '(co)datatype' -- eventual warnings (or errors) should be centralized in 'fp_bnf'
2013-11-06, by blanchet
removed dead code
2013-11-06, by blanchet
update docs
2013-11-06, by blanchet
take out possibility of moving corecursive calls past constructors -- this doesn't work in the general case
2013-11-06, by blanchet
took out loopy code
2013-11-06, by blanchet
take out even less aggressive generalization -- it's still too aggressive
2013-11-06, by blanchet
reverted too aggressive 7cb8442298f0
2013-11-06, by blanchet
generalize more aggressively
2013-11-06, by blanchet
avoid subtle failure in the presence of top sort
2013-11-05, by blanchet
tuning
2013-11-05, by blanchet
get mutually recursive maps as well
2013-11-05, by blanchet
tuned proofs in Approximation
2013-11-05, by hoelzl
fixed subtle name shadowing bug
2013-11-05, by blanchet
use right permutation in 'map2'
2013-11-05, by blanchet
stronger normalization, to increase n2m cache effectiveness
2013-11-05, by blanchet
make local theory operations non-pervasive (makes more intuitive sense)
2013-11-05, by blanchet
NEWS
2013-11-05, by hoelzl
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
2013-11-05, by hoelzl
generalize bdd_above/below_uminus to ordered_ab_group_add
2013-11-05, by hoelzl
restrict Limsup and Liminf to complete lattices
2013-11-05, by hoelzl
use INF and SUP on conditionally complete lattices in multivariate analysis
2013-11-05, by hoelzl
add SUP and INF for conditionally complete lattices
2013-11-05, by hoelzl
use bdd_above and bdd_below for conditionally complete lattices
2013-11-05, by hoelzl
generalize SUP and INF to the syntactic type classes Sup and Inf
2013-11-05, by hoelzl
added some N2M caching
2013-11-05, by blanchet
also generalize fixed types
2013-11-05, by blanchet
generalize types when synthetizing n2m (co)recursors, to facilitate reuse
2013-11-05, by blanchet
nicer error message in case of duplicates
2013-11-05, by blanchet
use int example like in the rest of IMP (instead of nat)
2013-11-05, by kleing
dropped dead code
2013-11-04, by haftmann
fact generalization and name consolidation
2013-11-04, by haftmann
streamlined setup of linear arithmetic
2013-11-04, by haftmann
make 'try0' return faster when invoked as part of 'try'
2013-11-04, by blanchet
careful with lists of different lengths
2013-11-04, by blanchet
split 'primrec_new' and 'primcorec' code (to ease bootstrapping, e.g. dependency on datatype 'String' in 'primcorec')
2013-11-04, by blanchet
better error handling
2013-11-04, by blanchet
more robust treatment of dead variables in n2m
2013-11-04, by traytel
more robust n2m w.r.t. 'let's
2013-11-04, by blanchet
tuning
2013-11-04, by blanchet
strengthened tactic
2013-11-04, by blanchet
made n2m code more robust w.r.t. advanced constructs (e.g. lambdas)
2013-11-04, by blanchet
handle constructor syntax in n2m primcorec
2013-11-04, by blanchet
typo
2013-11-04, by blanchet
made sugared 'coinduct' theorem construction n2m-proof
2013-11-04, by blanchet
moved code around
2013-11-04, by blanchet
tuning
2013-11-04, by blanchet
make code more robust w.r.t. applied/unapplied map (primrec vs. primcorec)
2013-11-04, by blanchet
conceal definition
2013-11-04, by blanchet
more exercises
2013-11-02, by nipkow
more exercises
2013-11-02, by nipkow
more simplification rules on unary and binary minus
2013-11-01, by haftmann
generate stable names for axioms
2013-10-31, by blanchet
purely algebraic foundation for even/odd
2013-10-31, by haftmann
moving generic lemmas out of theory parity, disregarding some unused auxiliary lemmas;
2013-10-31, by haftmann
explicit type class for modelling even/odd parity
2013-10-31, by haftmann
generalized of_bool conversion
2013-10-31, by haftmann
separated bit operations on type bit from generic syntactic bit operations
2013-10-31, by haftmann
restructed
2013-10-31, by haftmann
generalised lemma
2013-10-31, by haftmann
more lemmas on division
2013-10-31, by haftmann
more convenient place for a theory in solitariness
2013-10-31, by haftmann
consolidated clone theory
2013-10-31, by haftmann
more exercises
2013-10-31, by nipkow
tuned text
2013-10-30, by nipkow
inst_lift now fully instantiates context to avoid problems with loose bound variables
2013-10-29, by berghofe
include corecursive functions' arguments in callssss
2013-10-29, by panny
more exercises
2013-10-29, by nipkow
merged
2013-10-28, by nipkow
more exercises
2013-10-28, by nipkow
commented out vaporware
2013-10-27, by blanchet
more exercises
2013-10-26, by nipkow
tuning
2013-10-26, by blanchet
tuning
2013-10-26, by blanchet
tuned names (to make them independent from temporary naming convention used in characteristic theorems)
2013-10-26, by blanchet
align 'primrec_new' on 'primcorec' (+ got rid of one more 'dummyT')
2013-10-26, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
tip