Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
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.
conceal consts via name space, not tags;
2009-10-25, by wenzelm
allow name space entries to be "concealed" -- via binding/naming/local_theory;
2009-10-25, by wenzelm
switch to polyml-5.2.1 to see if it impacts performance;
2009-10-25, by wenzelm
merged
2009-10-25, by chaieb
Multivariate polynomials library over fields
2009-10-25, by chaieb
A theory of polynomials based on lists
2009-10-25, by chaieb
Add a quantifier elimination for parametric linear arithmetic over ordered fields (parameters are multivariate polynomials)
2009-10-25, by chaieb
merged
2009-10-25, by wenzelm
further changes due to the previous merge in the predicate compiler
2009-10-24, by bulwahn
merge -- imported from bulwahn d759e2728188;
2009-10-24, by wenzelm
removed tuple functions from the predicate compiler
2009-10-24, by bulwahn
improving the compilation with higher-order arguments in the predicate compiler
2009-10-24, by bulwahn
now the predicate compilere handles the predicate without introduction rules better as before
2009-10-24, by bulwahn
removed dead code; added examples
2009-10-24, by bulwahn
removed obsolete GeneratorPrem; clean-up after modularization; tuned
2009-10-24, by bulwahn
modularized the compilation in the predicate compiler
2009-10-24, by bulwahn
adapted parser for options in the predicate compiler
2009-10-24, by bulwahn
modifying the depth-limited compilation to be sound, but now throws an error undefined in case of hitting the depth limit in an negative context; cleaning up the examples
2009-10-24, by bulwahn
cleaning the signature of the predicate compiler core; renaming signature and structures to uniform long names
2009-10-24, by bulwahn
added skip_proof option; playing with compilation of depth-limited predicates
2009-10-24, by bulwahn
reinvestigating the compilation of the random computation in the predicate compiler
2009-10-24, by bulwahn
added option to generate random values to values command in the predicate compiler
2009-10-24, by bulwahn
commented out the random generator compilation in the example file
2009-10-24, by bulwahn
added option to execute depth-limited computations for the values command in the predicate compiler
2009-10-24, by bulwahn
renamed functions from sizelim to more natural name depth_limited for compilation of depth-limited search in the predicate compiler
2009-10-24, by bulwahn
simplified and improved compilation of depth-limited search in the predicate compiler
2009-10-24, by bulwahn
moved argument expected_modes into options; improved mode check to only check mode of the named predicate
2009-10-24, by bulwahn
removed unnecessary argument rpred in code_pred function
2009-10-24, by bulwahn
added option show_mode_inference; added splitting of conjunctions in expand_tuples
2009-10-24, by bulwahn
changed import_intros to handle parameters differently; changed handling of higher-order function compilation; reverted MicroJava change; tuned
2009-10-24, by bulwahn
further cleaning up
2009-10-24, by bulwahn
added option show_proof_trace
2009-10-24, by bulwahn
importing of polymorphic introduction rules with different schematic variable names
2009-10-24, by bulwahn
added option show_intermediate_results
2009-10-24, by bulwahn
continued cleaning up; moved tuple expanding to core
2009-10-24, by bulwahn
cleaned up debugging messages; added options to code_pred command
2009-10-24, by bulwahn
added first support for higher-order function translation
2009-10-24, by bulwahn
added to process higher-order arguments by adding new constants
2009-10-24, by bulwahn
cleaned up
2009-10-24, by bulwahn
added theory with alternative definitions for the predicate compiler; cleaned up examples
2009-10-24, by bulwahn
importing theorems correctly causes problems with mutual recursive predicates in the predicate compiler; must be discussed with Stefan first
2009-10-24, by bulwahn
higher-order arguments in different rules are fixed to one name in the predicate compiler
2009-10-24, by bulwahn
changed importing introduction rules to fix the same type variables in all introduction rules; improved mode analysis for partially applied relations; added test case; tuned
2009-10-24, by bulwahn
changed proof method to handle widen predicate in JinjaThreads
2009-10-24, by bulwahn
added further examples; added mode to code_pred command; tuned; some temporary things in Predicate_Compile_ex
2009-10-24, by bulwahn
processing of tuples in introduction rules
2009-10-24, by bulwahn
added a few tricky examples with tuples; added alternative introduction rules for some constants; corrected mode analysis with negation; improved fetching of definitions
2009-10-24, by bulwahn
developing an executable the operator
2009-10-24, by bulwahn
generalizing singleton with a default value
2009-10-24, by bulwahn
changed elimination preprocessing due to an error with a JinjaThread predicate
2009-10-24, by bulwahn
added test for higher-order function inductification; added debug messages
2009-10-24, by bulwahn
added filtering of case constants in the definition retrieval of the predicate compiler
2009-10-24, by bulwahn
extended core of predicate compiler to expand tuples in introduction rules
2009-10-24, by bulwahn
added tupled versions of examples for the predicate compiler
2009-10-24, by bulwahn
moved meta_fun_cong lemma into ML-file; tuned
2009-10-24, by bulwahn
merged
2009-10-25, by wenzelm
adapted Function_Lib (cf. b8cdd3d73022);
2009-10-25, by wenzelm
configuration flag "partials"
2009-10-24, by krauss
renamed auto_term.ML -> relation.ML
2009-10-23, by krauss
function package: more standard names for structures and files
2009-10-23, by krauss
renamed FundefDatatype -> Function_Fun
2009-10-23, by krauss
maintain position of formal entities via name space;
2009-10-24, by wenzelm
maintain explicit name space kind;
2009-10-24, by wenzelm
renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
2009-10-24, by wenzelm
eliminated separate stamp -- NameSpace.define/merge etc. ensure uniqueness already;
2009-10-24, by wenzelm
eliminated separate stamp -- NameSpace.define/merge etc. ensure uniqueness already;
2009-10-24, by wenzelm
eliminated separate stamp -- NameSpace.define/merge etc. ensure uniqueness already;
2009-10-24, by wenzelm
maintain abstract entry, with position, identity etc.;
2009-10-24, by wenzelm
tuned message;
2009-10-24, by wenzelm
import theory Nat here, which avoids duplicate definition of datatype_realizers (and thus allows to maintain fully authentic fact table);
2009-10-24, by wenzelm
markup for formal entities, with "def" or "ref" occurrences;
2009-10-24, by wenzelm
handle Sorts.CLASS_ERROR instead of arbitrary exceptions;
2009-10-24, by wenzelm
reactivated isatest on macbroy6 -- 3h later to avoid overlap with backup daemon;
2009-10-23, by wenzelm
merged
2009-10-23, by haftmann
turned off old quickcheck
2009-10-23, by haftmann
pat_completeness gets its own file
2009-10-23, by krauss
ignore error messages produced by ATPs
2009-10-23, by boehmes
merged
2009-10-23, by haftmann
renamed f_inv_onto_f to f_inv_into_f (cf. 764547b68538)
2009-10-23, by haftmann
restored accidentally deleted submultiset
2009-10-22, by haftmann
multiset operations with canonical argument order
2009-10-22, by haftmann
arg_types_of auxiliary function; using multiset operations
2009-10-22, by haftmann
merged
2009-10-23, by haftmann
close thm derivations explicitly
2009-10-22, by haftmann
Fix a duplicate abbreviation || in etc/symbols.
2009-10-23, by tbourke
made SML/NJ happy;
2009-10-22, by wenzelm
updated session name;
2009-10-22, by wenzelm
renamed f_inv_onto_f to f_inv_into_f (cf. 764547b68538);
2009-10-22, by wenzelm
merged
2009-10-22, by wenzelm
merged
2009-10-22, by wenzelm
merged
2009-10-21, by wenzelm
use plain Scan.repeat (NB: Scan.bulk is for cascading sources -- mostly interna use);
2009-10-21, by wenzelm
merged
2009-10-22, by wenzelm
explicit close_derivation
2009-10-22, by haftmann
merged
2009-10-22, by haftmann
map_range (and map_index) combinator
2009-10-22, by haftmann
dropped Datatype.distinct_simproc
2009-10-22, by haftmann
use Synchronized.assign to achieve actual immutable results;
2009-10-22, by wenzelm
support single-assigment variables -- based on magic RTS operations by David Matthews;
2009-10-22, by wenzelm
merged
2009-10-22, by boehmes
fixed permissions -- this is a script, not an executable
2009-10-22, by boehmes
inv_onto -> inv_into
2009-10-22, by nipkow
renamed "nitpick_const_xxx" attributes to "nitpick_xxx" and "nitpick_ind_intros" to "nitpick_intros"
2009-10-21, by blanchet
merged
2009-10-21, by blanchet
fixed the "expect" mechanism of Refute in the face of timeouts
2009-10-21, by blanchet
removed "nitpick_const_simp" attribute from Record's "simps";
2009-10-21, by blanchet
merged
2009-10-21, by haftmann
more accurate removal
2009-10-21, by haftmann
merged
2009-10-21, by haftmann
curried inter as canonical list operation (beware of argument order)
2009-10-21, by haftmann
merged
2009-10-21, by boehmes
proper handling of single literal case,
2009-10-21, by boehmes
Removed the hard-wired white list of theorems for sledgehammer
2009-10-21, by paulson
merged
2009-10-21, by paulson
Some new lemmas concerning sets
2009-10-20, by paulson
merged
2009-10-21, by haftmann
curried union as canonical list operation
2009-10-21, by haftmann
tuned ML import
2009-10-21, by haftmann
removed old-style \ and \\ infixes
2009-10-21, by haftmann
merged
2009-10-21, by haftmann
dropped redundant gen_ prefix
2009-10-21, by haftmann
replaced old_style infixes eq_set, subset, union, inter and variants by generic versions
2009-10-20, by haftmann
find_theorems: better handling of abbreviations (by Timothy Bourke)
2009-10-21, by kleing
standardized basic operations on type option;
2009-10-21, by wenzelm
eliminated THENL -- use THEN RANGE;
2009-10-20, by wenzelm
tuned;
2009-10-20, by wenzelm
fixed SML/NJ toplevel pp;
2009-10-20, by wenzelm
backpatching of structure Proof and ProofContext -- avoid odd aliases;
2009-10-20, by wenzelm
tuned;
2009-10-20, by wenzelm
uniform use of Integer.min/max;
2009-10-20, by wenzelm
modernized session SET_Protocol;
2009-10-20, by wenzelm
modernized session Metis_Examples;
2009-10-20, by wenzelm
modernized session Isar_Examples;
2009-10-20, by wenzelm
tuned header;
2009-10-20, by wenzelm
more accurate dependencies for HOL-SMT, which is a session with image;
2009-10-20, by wenzelm
removed unused map_force;
2009-10-20, by wenzelm
Removal of the unused atpset concept, the atp attribute and some related code.
2009-10-20, by paulson
additional schematic rules for Z3's rewrite rule
2009-10-20, by boehmes
merged
2009-10-20, by nipkow
added Hilbert_Choice section
2009-10-20, by nipkow
merged
2009-10-20, by boehmes
eliminated extraneous wrapping of public records,
2009-10-20, by boehmes
proper exceptions instead of unhandled partiality
2009-10-20, by boehmes
footnote: inv via inv_onto
2009-10-20, by nipkow
added inv_def for compatibility as a lemma
2009-10-20, by nipkow
slightly less context-sensitive settings;
2009-10-20, by wenzelm
merged
2009-10-20, by wenzelm
corrected paths to certificates,
2009-10-20, by boehmes
added proof reconstructon for Z3,
2009-10-20, by boehmes
merged
2009-10-20, by wenzelm
merged
2009-10-20, by haftmann
more accurate checkpoints
2009-10-20, by haftmann
dropped lazy code equations
2009-10-19, by haftmann
CONTRIBUTORS
2009-10-19, by haftmann
always qualify NJ's old List.foldl/foldr in Isabelle/ML;
2009-10-19, by wenzelm
eliminated duplicate fold1 -- beware of argument order!
2009-10-19, by wenzelm
uniform use of Integer.add/mult/sum/prod;
2009-10-19, by wenzelm
Removed dead code in function mk_deftab.
2009-10-19, by berghofe
Removed unneeded reference to inv_def.
2009-10-19, by berghofe
Replaced inv by the_inv_onto.
2009-10-19, by berghofe
Renamed inv to the_inv and turned it into an abbreviation (based on the_inv_onto).
2009-10-19, by berghofe
fixed proof (cf. d1d4d7a08a66);
2009-10-18, by wenzelm
removed disjunctive group cancellation -- provers run independently;
2009-10-18, by wenzelm
tuned;
2009-10-18, by wenzelm
removed some unreferenced material;
2009-10-18, by wenzelm
merged
2009-10-18, by nipkow
certificates for sos
2009-10-18, by nipkow
merged
2009-10-18, by nipkow
added sums of squares for standard deviation
2009-10-18, by nipkow
merged
2009-10-18, by nipkow
Inv -> inv_onto, inv abbr. inv_onto UNIV.
2009-10-18, by nipkow
disable indent-tabs-mode in Proof General / Emacs;
2009-10-18, by wenzelm
merged
2009-10-17, by wenzelm
made SML/NJ happy;
2009-10-17, by wenzelm
Merged.
2009-10-17, by ballarin
Finished revisions of locales tutorial.
2009-10-17, by ballarin
Changed part of the examples to int.
2009-10-15, by ballarin
Save current state of locales tutorial.
2009-10-15, by ballarin
Observe order of declaration when printing registrations.
2009-10-15, by ballarin
disable sunbroy2 for now;
2009-10-17, by wenzelm
tuned/moved divide_and_conquer';
2009-10-17, by wenzelm
tuned;
2009-10-17, by wenzelm
removed separate record_quick_and_dirty_sensitive;
2009-10-17, by wenzelm
simplified tactics;
2009-10-17, by wenzelm
eliminated old List.foldr and OldTerm operations;
2009-10-17, by wenzelm
removed unused names;
2009-10-17, by wenzelm
misc tuning and simplification;
2009-10-17, by wenzelm
less pervasive names;
2009-10-17, by wenzelm
operations of structure Skip_Proof (formerly SkipProof) no longer require quick_and_dirty mode;
2009-10-17, by wenzelm
Method.cheating: check quick_and_dirty here;
2009-10-17, by wenzelm
tuned;
2009-10-17, by wenzelm
Unsynchronized.set etc.;
2009-10-17, by wenzelm
indicate CRITICAL nature of various setmp combinators;
2009-10-17, by wenzelm
ISABELLE_TOOL;
2009-10-17, by wenzelm
tuned signature;
2009-10-17, by wenzelm
merged
2009-10-17, by wenzelm
merged
2009-10-17, by nipkow
added the_inv_onto
2009-10-17, by nipkow
eliminated hard tabulators, guessing at each author's individual tab-width;
2009-10-17, by wenzelm
removed obsolete old goal command;
2009-10-17, by wenzelm
legacy Drule.standard is no longer pervasive;
2009-10-17, by wenzelm
explicitly qualify Drule.standard;
2009-10-17, by wenzelm
tuned white space;
2009-10-16, by wenzelm
local channels for tracing/debugging;
2009-10-16, by wenzelm
made SML/NJ happy;
2009-10-16, by wenzelm
sunbroy2: back to single-threaded mode for now -- deadlock in Poly/ML 5.3-SVN-900;
2009-10-15, by wenzelm
replaced String.concat by implode;
2009-10-15, by wenzelm
space_implode;
2009-10-15, by wenzelm
normalized aliases of Output operations;
2009-10-15, by wenzelm
eliminated slightly odd get/set operations in favour of Unsynchronized.ref;
2009-10-15, by wenzelm
natural argument order for prover;
2009-10-15, by wenzelm
ATP_Manager.get_prover: canonical argument order;
2009-10-15, by wenzelm
tuned proof (via atp_minimized);
2009-10-15, by wenzelm
sort_strings (cf. Pure/library.ML);
2009-10-15, by wenzelm
clarified File.platform_path vs. File.shell_path;
2009-10-15, by wenzelm
exported File.shell_quote;
2009-10-15, by wenzelm
misc tuning and recovery of Isabelle coding style;
2009-10-15, by wenzelm
eliminated extraneous wrapping of public records;
2009-10-15, by wenzelm
tuned signature;
2009-10-15, by wenzelm
renamed functor HeapFun to Heap;
2009-10-15, by wenzelm
misc tuning and clarification;
2009-10-15, by wenzelm
structure ATP_Manager: eliminated slightly odd get/set operations in favour of Unsynchronized.ref;
2009-10-15, by wenzelm
modernized structure names;
2009-10-14, by wenzelm
show direct GC time (which is included in CPU time);
2009-10-14, by wenzelm
eliminated obsolete C/flip combinator;
2009-10-14, by wenzelm
added List.nth
2009-10-14, by nipkow
tuned make parameters for sunbroy2;
2009-10-14, by wenzelm
accomodate old version of "tail", e.g. on sunbroy2;
2009-10-14, by wenzelm
settings for parallel experimental Poly/ML 5.3;
2009-10-14, by wenzelm
sharpened name
2009-10-14, by haftmann
more explicit notion of canonized code equations
2009-10-14, by haftmann
more explicit notion of canonized code equations
2009-10-14, by haftmann
tuned whitespace
2009-10-14, by haftmann
tuned whitespace
2009-10-14, by haftmann
dropped Code_Printer prefix where feasible; fixed whitespace issues; more coherent terminology
2009-10-14, by haftmann
merged
2009-10-13, by haftmann
deactivated Datatype.distinct_simproc
2009-10-13, by haftmann
dropped Datatype.distinct_simproc; tuned
2009-10-13, by haftmann
order conjunctions to be printed without parentheses
2009-10-13, by hoelzl
approximation now fails earlier when using interval splitting; value [approximate] now supports bounded variables; renamed Var -> Atom for better readability
2009-10-13, by hoelzl
merged
2009-10-13, by haftmann
added add_tyconames; tuned
2009-10-12, by haftmann
merged
2009-10-13, by haftmann
more appropriate abstraction over distinctness rules
2009-10-13, by haftmann
merged
2009-10-12, by haftmann
intro_base_names combinator
2009-10-12, by haftmann
merged
2009-10-12, by haftmann
dropped dist_ss
2009-10-12, by haftmann
merged
2009-10-12, by haftmann
added is_IVar
2009-10-12, by haftmann
factored out Code_Printer.aux_params
2009-10-12, by haftmann
dropped rule duplicates
2009-10-12, by haftmann
less non-standard combinators
2009-10-12, by haftmann
nth replaces List.nth
2009-10-12, by haftmann
dropped redundancy
2009-10-12, by haftmann
dropped dead code
2009-10-12, by haftmann
using distinct rules directly
2009-10-12, by haftmann
simplified proof
2009-10-09, by haftmann
dropped simproc_dist formally
2009-10-09, by haftmann
tuned order of lemmas
2009-10-09, by haftmann
term styles also cover antiquotations term_type and typeof
2009-10-09, by haftmann
merged
2009-10-09, by haftmann
lookup for datatype constructors considers type annotations to resolve overloading
2009-10-08, by haftmann
added group_stmts
2009-10-08, by haftmann
moved labelled_name to code_thingol
2009-10-08, by haftmann
updated generated documentation
2009-10-08, by haftmann
corrected syntax diagrams for styles
2009-10-08, by haftmann
new generalized concept for term styles
2009-10-08, by haftmann
generalized term styles: transformations may depend on arguments; modernized term_style module; antiquotations thm, prop and term accepting term styles
2009-10-07, by haftmann
isatest: store test identifiers
2009-10-08, by krauss
tuned proofs
2009-10-07, by haftmann
added bot_boolE, top_boolI
2009-10-07, by haftmann
do not use Locale.add_registration_eqs any longer
2009-10-07, by haftmann
Inf/Sup now purely syntactic
2009-10-07, by haftmann
merged
2009-10-06, by haftmann
inf/sup1/2_iff are mere duplicates of underlying definitions: dropped
2009-10-06, by haftmann
merged
2009-10-06, by haftmann
added Coset as constructor
2009-10-06, by haftmann
sets and cosets
2009-10-06, by haftmann
added syntactic Inf and Sup
2009-10-06, by haftmann
merged
2009-10-05, by paulson
New lemmas connected with the reals and infinite series
2009-10-05, by paulson
New facts about domain and range in
2009-10-05, by paulson
merged
2009-10-05, by haftmann
experimental de-facto abolishment of distinctness limit
2009-10-05, by haftmann
tuned handling of type variable names further
2009-10-05, by haftmann
variables in type schemes must be renamed simultaneously with variables in equations
2009-10-05, by haftmann
explicitly unsynchronized
2009-10-05, by haftmann
explicitly unsynchronized
2009-10-05, by haftmann
recovered support for Spass: re-enabled writing problems in DFG format
2009-10-04, by boehmes
avoid exception Option: only apply "the" if needed
2009-10-04, by boehmes
merged
2009-10-04, by nipkow
atp_minimal using chain_ths again
2009-09-30, by Philipp Meyer
merged
2009-10-03, by boehmes
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
2009-10-03, by boehmes
eliminated dead code;
2009-10-02, by wenzelm
eliminated dead code and redundant parameters;
2009-10-02, by wenzelm
eliminated dead code;
2009-10-02, by wenzelm
replaced Proof.get_goal state by Proof.flat_goal state, which provides the standard view on goals for (semi)automated tools;
2009-10-02, by wenzelm
replaced Proof.get_goal state by Proof.flat_goal state, which provides the standard view on goals for (semi)automated tools;
2009-10-02, by wenzelm
Refute.refute_goal: goal addressing from 1 as usual;
2009-10-02, by wenzelm
Refute.refute_goal: canonical goal addresses from 1 (renamed from refute_subgoal to clarify change in semantics);
2009-10-02, by wenzelm
clarified Proof.refine_insert -- always "refine" to apply standard method treatment (of conjunctions);
2009-10-02, by wenzelm
misc tuning and simplification;
2009-10-02, by wenzelm
macbroy2: bigger jobs first, to avoid danger of swapping during daytime;
2009-10-02, by wenzelm
less ambitious heap settings;
2009-10-02, by wenzelm
merged
2009-10-02, by haftmann
merged
2009-10-01, by haftmann
proper merge of interpretation equations
2009-10-01, by haftmann
merged
2009-10-02, by wenzelm
Merged again.
2009-10-01, by ballarin
Merged.
2009-10-01, by ballarin
News entry: inheritance of mixins; print_interps.
2009-10-01, by ballarin
Avoid administrative overhead for identity mixins.
2009-10-01, by ballarin
tuned;
2009-10-01, by wenzelm
moved cache_conv to src/Pure/conv.ML, use Thm.cterm_cache;
2009-10-01, by wenzelm
added Ctermtab, cterm_cache, thm_cache;
2009-10-01, by wenzelm
added term_cache;
2009-10-01, by wenzelm
Concurrently cached values.
2009-10-01, by wenzelm
tuned header;
2009-10-01, by wenzelm
core_sos_tac: SUBPROOF body operates on subgoal 1;
2009-10-01, by wenzelm
merged
2009-10-01, by wenzelm
updated generated files;
2009-10-01, by wenzelm
enable slow-motion mode to accomodate unsynchronized refs within theory sources;
2009-10-01, by wenzelm
avoid unsynchronized refs within theory sources;
2009-10-01, by wenzelm
explicitly Unsynchronized;
2009-10-01, by wenzelm
additional fixes in normarith.ML due to FuncFun and FuncUtil changes
2009-10-01, by Philipp Meyer
changed core_sos_tac to use SUBPROOF
2009-10-01, by Philipp Meyer
replaced and tuned uses of foldr1
2009-09-30, by Philipp Meyer
tuned FuncFun and FuncUtil structure in positivstellensatz.ML
2009-09-30, by Philipp Meyer
removed opening of structures
2009-09-22, by Philipp Meyer
merged
2009-10-01, by wenzelm
merged
2009-10-01, by nipkow
merged
2009-10-01, by nipkow
made spass additional default prover
2009-10-01, by nipkow
merged
2009-10-01, by paulson
Proved a new theorem: nat_to_nat2_inj
2009-10-01, by paulson
turned unsynchronized ref into synchronized var
2009-10-01, by boehmes
merged
2009-10-01, by nipkow
resolved conflict
2009-10-01, by nipkow
record max lemmas used
2009-10-01, by nipkow
Lazy evaluation with memoing (sequential version).
2009-10-01, by wenzelm
more official status of sequential implementations;
2009-10-01, by wenzelm
separate concurrent/sequential versions of lazy evaluation;
2009-10-01, by wenzelm
added Task_Queue.depend (again) -- light-weight version for transitive graph;
2009-10-01, by wenzelm
handle Pattern.MATCH, not arbitrary exceptions;
2009-10-01, by wenzelm
more precise dependencies;
2009-10-01, by wenzelm
eliminated redundant parameters;
2009-10-01, by wenzelm
back to simple fold_body_thms and fulfill_proof/thm_proof (reverting a900d3cd47cc) -- the cycle check is implicit in the future computation of join_proofs;
2009-10-01, by wenzelm
avoid mixed l/r infixes, which do not work in some versions of SML;
2009-10-01, by wenzelm
tuned;
2009-10-01, by wenzelm
merged
2009-10-01, by wenzelm
explicitly Unsynchronized
2009-10-01, by haftmann
Merged.
2009-10-01, by ballarin
Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
2009-09-29, by ballarin
Archive registrations by external view.
2009-09-27, by ballarin
Stricter test: raise error if registration generates duplicate theorem.
2009-09-26, by ballarin
Explicit management of registration mixins.
2009-09-19, by ballarin
Improved comments and api names.
2009-08-19, by ballarin
eliminated dead code, redundant bindings and parameters;
2009-10-01, by wenzelm
misc tuning and simplification;
2009-10-01, by wenzelm
eliminated dead code;
2009-09-30, by wenzelm
eliminated dead code;
2009-09-30, by wenzelm
Sorts.of_sort_derivation: no pp here;
2009-09-30, by wenzelm
eliminated redundant bindings;
2009-09-30, by wenzelm
actually perform Isar_Document.init on startup;
2009-09-30, by wenzelm
eliminated dead code;
2009-09-30, by wenzelm
removed dead code;
2009-09-30, by wenzelm
handle Type.TYPE_MATCH, not arbitrary exceptions;
2009-09-30, by wenzelm
removed redundant Sign.certify_prop, use Sign.cert_prop instead;
2009-09-30, by wenzelm
PARALLEL_GOALS: proper scope for exception FAILED, with dummy argument to prevent its interpretation as variable;
2009-09-30, by wenzelm
actually export unit parser;
2009-09-30, by wenzelm
eliminated dead code;
2009-09-30, by wenzelm
eliminated redundant parameters;
2009-09-30, by wenzelm
eliminated redundant bindings;
2009-09-30, by wenzelm
merged
2009-09-30, by haftmann
moved lemmas about sup on bool to Lattices.thy
2009-09-30, by haftmann
moved lemmas about sup on bool to Lattices.thy
2009-09-30, by haftmann
tuned proofs
2009-09-30, by haftmann
tuned headings
2009-09-30, by haftmann
report unreferenced ids;
2009-09-30, by wenzelm
tuned whitespace;
2009-09-30, by wenzelm
more uniform treatment of structure Unsynchronized in ML bootstrap phase;
2009-09-30, by wenzelm
merged
2009-09-30, by haftmann
mandatory prefix where appropriate
2009-09-30, by haftmann
mandatory prefix where appropriate
2009-09-30, by haftmann
tuned whitespace
2009-09-30, by haftmann
replaced chained_goal by slightly more appropriate flat_goal;
2009-09-30, by wenzelm
made SML/NJ happy;
2009-09-30, by wenzelm
added chained_goal, which presents the goal thm as seen by semi-structured methods;
2009-09-30, by wenzelm
tuned;
2009-09-29, by wenzelm
removed dead/duplicate code;
2009-09-29, by wenzelm
aliases for Thomas Sewell;
2009-09-29, by wenzelm
modernized Balanced_Tree;
2009-09-29, by wenzelm
replaced meta_iffD2 by existing Drule.equal_elim_rule2;
2009-09-29, by wenzelm
tuned header;
2009-09-29, by wenzelm
Thomas Sewell, NICTA: more efficient HOL/record implementation;
2009-09-29, by wenzelm
tuned whitespace -- recover basic Isabelle conventions;
2009-09-29, by wenzelm
merged
2009-09-29, by wenzelm
Merge with isabelle dev changes.
2009-09-29, by Thomas Sewell
Replace OldTerm.term_vars with Term.add_vars in named_cterm_instantiate.
2009-09-29, by Thomas Sewell
Avoid a possible variable name conflict in instantiating a theorem.
2009-09-28, by Thomas Sewell
Fix unescaped expressions breaking latex output in Record.thy
2009-09-28, by Thomas Sewell
Merge record patch with updates from isabelle mainline.
2009-09-28, by Thomas Sewell
Avoid record-inner constants in polymorphic definitions in Bali
2009-09-25, by Thomas Sewell
Merge with changes from isabelle dev repository.
2009-09-24, by Thomas Sewell
Initial response to feedback from Norbert, Makarius on record patch
2009-09-23, by tsewell
Branch merge for isabelle mainline updates.
2009-09-22, by Thomas Sewell
Branch merge with updates from mainline isabelle.
2009-09-17, by Thomas Sewell
Implement previous fix (don't duplicate ext_def) correctly.
2009-09-11, by Thomas Sewell
There's no particular reason to duplicate the extension
2009-09-11, by Thomas Sewell
Merged with mainline changes.
2009-09-11, by Thomas Sewell
Adjust some documentation.
2009-09-11, by Thomas Sewell
Simplification of various aspects of the IsTuple component
2009-09-10, by Thomas Sewell
Record patch imported and working.
2009-09-10, by Thomas Sewell
Initial attempt at porting record update to repository Isabelle.
2009-08-27, by tsewell
Synchronized and Unsynchronized;
2009-09-29, by wenzelm
hide "ref" by default, to enforce excplicit indication as Unsynchronized;
2009-09-29, by wenzelm
explicit indication of Unsynchronized.ref;
2009-09-29, by wenzelm
open_unsynchronized for interactive Isar loop;
2009-09-29, by wenzelm
explicit indication of Unsynchronized.ref;
2009-09-29, by wenzelm
Raw ML references as unsynchronized state variables.
2009-09-29, by wenzelm
Dummy version of state variables -- plain refs for sequential access.
2009-09-28, by wenzelm
reactivated at-sml-dev-e;
2009-09-28, by wenzelm
misc tuning and modernization;
2009-09-28, by wenzelm
moved generic cong_tac from HOL/Tools/datatype_aux.ML to Tools/cong_tac.ML, proper subgoal selection (failure, not exception);
2009-09-28, by wenzelm
merged
2009-09-28, by wenzelm
less auxiliary functions
2009-09-28, by haftmann
tuned
2009-09-28, by haftmann
shared code between rep_datatype and datatype
2009-09-28, by haftmann
further unification of datatype and rep_datatype
2009-09-28, by haftmann
avoid compound fields in datatype info record
2009-09-28, by haftmann
fold_body_thms: pass pthm identifier;
2009-09-28, by wenzelm
tuned internal source structure;
2009-09-28, by wenzelm
added fork_deps_pri;
2009-09-28, by wenzelm
merged
2009-09-28, by haftmann
explicit pointless checkpoint
2009-09-28, by haftmann
emerging common infrastructure for datatype and rep_datatype
2009-09-27, by haftmann
streamlined rep_datatype further
2009-09-27, by haftmann
simplified rep_datatype
2009-09-27, by haftmann
more appropriate order of field in dt_info
2009-09-27, by haftmann
re-established reasonable inner outline for module
2009-09-27, by haftmann
merged
2009-09-27, by wenzelm
adjusted to changes in datatype package
2009-09-27, by haftmann
merged
2009-09-27, by haftmann
dropped dead code
2009-09-27, by haftmann
registering split rules and projected induction rules; ML identifiers more close to Isar theorem names
2009-09-27, by haftmann
fold_body_thms/join_bodies: explicitly check for cyclic theorem references;
2009-09-27, by wenzelm
tuned;
2009-09-27, by wenzelm
reachable: recovered reverse post-order (lost in 73ad4884441f), which is expected for all_preds/all_succs and required for topological_order;
2009-09-27, by wenzelm
merged
2009-09-25, by paulson
New lemmas involving the real numbers, especially limits and series
2009-09-25, by paulson
NEWS; corrected spelling
2009-09-25, by haftmann
merged
2009-09-25, by haftmann
simplified proof
2009-09-23, by haftmann
removed potentially dangerous rules from pred_set_conv
2009-09-23, by haftmann
explicitly hide empty, inter, union
2009-09-23, by haftmann
merged
2009-09-23, by haftmann
merged
2009-09-23, by haftmann
merged
2009-09-23, by haftmann
inf/sup_absorb are no default simp rules any longer
2009-09-23, by haftmann
merged
2009-09-22, by haftmann
merged
2009-09-21, by haftmann
adapted proof
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proofs
2009-09-21, by haftmann
tuned header
2009-09-21, by haftmann
added note on simp rules
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proof; tuned headers
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proofs; be more cautios wrt. default simp rules
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proofs
2009-09-21, by haftmann
merged
2009-09-19, by haftmann
inter and union are mere abbreviations for inf and sup
2009-09-19, by haftmann
merged
2009-09-24, by haftmann
lemma relating fold1 and foldl; code_unfold rules for Inf_fin, Sup_fin, Min, Max, Inf, Sup
2009-09-24, by haftmann
subsumed by more general setup in List.thy
2009-09-24, by haftmann
idempotency case for fold1
2009-09-24, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip