Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+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.
clarified signature: full dependency graph;
2019-09-01, by wenzelm
merged
2019-08-31, by wenzelm
more scalable isabelle dump (and derivatives): mark individual theories to share common data in ML;
2019-08-29, by wenzelm
tuned signature;
2019-08-29, by wenzelm
merged
2019-08-29, by nipkow
simplified proofs
2019-08-29, by nipkow
more rules for ordered real vector spaces
2019-08-29, by haftmann
simplified setup
2019-08-29, by nipkow
tuned proof
2019-08-29, by nipkow
merged
2019-08-28, by wenzelm
enable share_common_data for "isabelle dump" and its derivatives (e.g. "isabelle mmt_import"): this has the potential to reduce ML heap size considerably, after initial command definitions;
2019-08-28, by wenzelm
support for share_common_data after define_command and before actual update: this affects string particles of command tokens;
2019-08-28, by wenzelm
more scalable -- less ML heap requirements;
2019-08-28, by wenzelm
tuned whitespace;
2019-08-28, by wenzelm
Integrate locale activation fallback diagnostics with 'trace_locales'.
2019-08-28, by ballarin
entry point for analysis without integration theory
2019-08-28, by immler
removed Brouwer_Fixpoint from imports of Derivative
2019-08-28, by immler
removed unused lemma, generalized, reduced dependencies
2019-08-27, by immler
fixed typo
2019-08-27, by immler
moved lemmas; reduced dependencies of Lipschitz
2019-08-27, by immler
explicit instance real::ordered_real_vector before subclass in ordered_euclidean_space
2019-08-27, by immler
merged
2019-08-27, by nipkow
moved lemmas
2019-08-27, by nipkow
moved basic theorem
2019-08-27, by immler
proper positions for 'termination' command (see also 5549e686d6ac);
2019-08-27, by wenzelm
tuned names -- proper scopes;
2019-08-27, by wenzelm
added system option "execution_eager": potentially reduce resource requires for "isabelle mmt_import" (smaller subgraphs are finished and disposed earlier);
2019-08-26, by wenzelm
proper positions for 'termination' command instead of original 'function' command, e.g. relevant for isabelle mmt_import;
2019-08-25, by wenzelm
Tracing of locale activation.
2019-08-24, by ballarin
tuned
2019-08-23, by nipkow
always export Pure proofs;
2019-08-23, by wenzelm
clarified 'thm_deps' command;
2019-08-23, by wenzelm
more compact: avoid pointless PThm rudiments;
2019-08-23, by wenzelm
clarified signature: prefer total operations;
2019-08-23, by wenzelm
proper graph traversal: avoid multiple visit of unnamed nodes;
2019-08-21, by wenzelm
more scalable: avoid huge intermediate XML elems;
2019-08-21, by wenzelm
more scalable buffer: produce compact chunks on the fly, avoid too many small particles that might congest heap management;
2019-08-21, by wenzelm
NEWS;
2019-08-20, by wenzelm
merged
2019-08-20, by wenzelm
export thm_deps;
2019-08-20, by wenzelm
proper theory context;
2019-08-20, by wenzelm
clarified thm_id vs. thm_node/thm: retain theory_name;
2019-08-20, by wenzelm
clarified signature;
2019-08-20, by wenzelm
tuned;
2019-08-20, by wenzelm
unused (see 095dadc62bb5);
2019-08-20, by wenzelm
tuned;
2019-08-20, by wenzelm
tuned signature;
2019-08-20, by wenzelm
clarified modules;
2019-08-20, by wenzelm
clarified modules;
2019-08-20, by wenzelm
tuned;
2019-08-20, by wenzelm
clarified signature;
2019-08-20, by wenzelm
tuned
2019-08-20, by nipkow
tuned
2019-08-20, by nipkow
merged
2019-08-20, by nipkow
tuned
2019-08-20, by nipkow
merged
2019-08-19, by wenzelm
clarified signature;
2019-08-19, by wenzelm
clarified export of axioms and theorems (identified derivations instead of projected facts);
2019-08-19, by wenzelm
tuned signature;
2019-08-19, by wenzelm
back to uniform serial (reverting 913b4afb6ac2): this allows to treat derivation id like name space entity id;
2019-08-19, by wenzelm
module Thm_Name for Isabelle/Scala;
2019-08-19, by wenzelm
tuned;
2019-08-19, by wenzelm
clarified modules;
2019-08-19, by wenzelm
tuned;
2019-08-19, by wenzelm
tuned
2019-08-19, by nipkow
tuned names
2019-08-19, by nipkow
clarified signature;
2019-08-17, by wenzelm
discontinued peek_status: unused and not clearly defined;
2019-08-17, by wenzelm
more documentation on oracles;
2019-08-17, by wenzelm
proper theory context for global props;
2019-08-17, by wenzelm
more thorough check, using full dependency graph of finished proofs;
2019-08-17, by wenzelm
added ML antiquotation @{oracle_name};
2019-08-17, by wenzelm
more robust, notably for open_proof of unnamed derivation;
2019-08-17, by wenzelm
tuned comments;
2019-08-17, by wenzelm
NEWS;
2019-08-17, by wenzelm
more accurate proposition for cheat_tac (command 'sorry');
2019-08-17, by wenzelm
added command 'thm_oracles';
2019-08-17, by wenzelm
clarified type for recorded oracles;
2019-08-17, by wenzelm
unused;
2019-08-17, by wenzelm
clarified signature;
2019-08-17, by wenzelm
clarified modules;
2019-08-17, by wenzelm
clarified lookup operations: more scalable for multiple retrieval;
2019-08-17, by wenzelm
clarified signature;
2019-08-17, by wenzelm
merged
2019-08-16, by wenzelm
maintain thm_name vs. derivation_id for global facts;
2019-08-16, by wenzelm
clarified identity of PThm nodes: do not reuse old id after renaming -- enforce uniqueness of substructures;
2019-08-16, by wenzelm
clarified signature;
2019-08-16, by wenzelm
Fixed brace matching (plus some whitespace cleanup)
2019-08-16, by paulson
merged
2019-08-16, by paulson
new material on eqiintegrable functions, etc.
2019-08-16, by paulson
clarified treatment of individual theorems;
2019-08-16, by wenzelm
tuned signature;
2019-08-16, by wenzelm
clarified signature;
2019-08-16, by wenzelm
clarified derivation_name vs. raw_derivation_name;
2019-08-16, by wenzelm
merged
2019-08-15, by wenzelm
more careful treatment of hidden type variable names: smash before zero_var_indexes to get standard enumeration;
2019-08-15, by wenzelm
more careful treatment of standard_vars: rename apart from existing frees and avoid approximative Name.declared, proper application of unvarifyT within terms of proof;
2019-08-15, by wenzelm
support Export_Theory.read_proof, based on theory_name and serial;
2019-08-15, by wenzelm
clarified PThm: theory_name simplifies retrieval from exports;
2019-08-15, by wenzelm
Indexname.toString according to string_of_vname' in ML;
2019-08-15, by wenzelm
clarified type Indexname, with plain value Int;
2019-08-15, by wenzelm
more complete pattern match;
2019-08-15, by wenzelm
export facts with reconstructed proof term (if possible), but its PThm boxes need to be collected separately;
2019-08-15, by wenzelm
support for (fully reconstructed) proof terms in Scala;
2019-08-15, by wenzelm
new material; rotated premises of Lim_transform_eventually
2019-08-15, by paulson
clarified name context for abstractions -- in contrast to 367e60d9aa1b and Term.variant_frees (*as they are printed :-*);
2019-08-14, by wenzelm
tuned;
2019-08-14, by wenzelm
uniform standard_vars for terms and proof terms;
2019-08-14, by wenzelm
treat simproc results as atomic -- more compact proof terms;
2019-08-14, by wenzelm
tuned;
2019-08-13, by wenzelm
minor performance tuning;
2019-08-13, by wenzelm
NEWS and example for Theory.join_theory;
2019-08-13, by wenzelm
tuned whitespace;
2019-08-13, by wenzelm
more compact proof terms;
2019-08-13, by wenzelm
more documentation;
2019-08-13, by wenzelm
added SUBPROOFS / "subproofs" method combinator, for more compact proofterms;
2019-08-13, by wenzelm
clarified modules;
2019-08-13, by wenzelm
merged
2019-08-12, by wenzelm
more compact proof terms;
2019-08-12, by wenzelm
more robust -- notably for metis, which tends to accumulate tpairs;
2019-08-12, by wenzelm
tuned -- avoid shadowing of ML names;
2019-08-12, by wenzelm
tuned;
2019-08-12, by wenzelm
more compact proof terms;
2019-08-12, by wenzelm
tuned;
2019-08-12, by wenzelm
tuned;
2019-08-12, by wenzelm
tuned -- eliminated unused parameters;
2019-08-12, by wenzelm
more direct/compact export of proof terms;
2019-08-12, by wenzelm
output physical_stderr, e.g. for low-level debugging;
2019-08-12, by wenzelm
tuned;
2019-08-12, by wenzelm
do not open ML structures;
2019-08-12, by wenzelm
tuned;
2019-08-12, by wenzelm
misc tuning -- slightly more readable;
2019-08-12, by wenzelm
simplified defs (thanks to Mohammad)
2019-08-12, by nipkow
record sort constraints unconditionally: minimal performance implications;
2019-08-11, by wenzelm
more careful export of unnamed proof boxes: avoid duplicates via memoing;
2019-08-10, by wenzelm
tuned signature;
2019-08-10, by wenzelm
export each PThm node separately: slightly more scalable;
2019-08-10, by wenzelm
allow duplicate exports via strict = false;
2019-08-10, by wenzelm
tuned message;
2019-08-10, by wenzelm
more positions;
2019-08-10, by wenzelm
more positions;
2019-08-10, by wenzelm
tuned;
2019-08-09, by wenzelm
formal position for PThm nodes;
2019-08-09, by wenzelm
clarified ML types;
2019-08-09, by wenzelm
proper treatment of body oracles, outside of recursion into thms graph;
2019-08-09, by wenzelm
prefer named lemmas -- more compact proofterms;
2019-08-08, by wenzelm
prefer named lemmas -- more compact proofterms;
2019-08-08, by wenzelm
tuned whitespace -- slightly more readable;
2019-08-08, by wenzelm
clarified signature: fewer warnings in ML IDE;
2019-08-08, by wenzelm
tuned;
2019-08-08, by wenzelm
prefer named lemmas -- more compact proofterms;
2019-08-07, by wenzelm
more compact proofterms;
2019-08-07, by wenzelm
eliminated pointless comments;
2019-08-07, by wenzelm
clarified proofterms;
2019-08-07, by wenzelm
more robust and convenient treatment of implicit context;
2019-08-07, by wenzelm
removed junk (cf. fa933b98d64d);
2019-08-07, by wenzelm
explicit check of left-over constraints from different theory, e.g. due to lack of Thm.trim_context;
2019-08-07, by wenzelm
more careful treatment of implicit context;
2019-08-07, by wenzelm
more careful treatment of implicit context;
2019-08-07, by wenzelm
proper build options;
2019-08-07, by wenzelm
merged
2019-08-06, by wenzelm
backed out changeset 1b8858f4c393: odd problems e.g. in CAVA_LTL_Modelchecker;
2019-08-06, by wenzelm
more careful treatment of implicit context;
2019-08-06, by wenzelm
clarified signature;
2019-08-06, by wenzelm
more robust and convenient treatment of implicit context;
2019-08-06, by wenzelm
clarified context: proper transfer;
2019-08-06, by wenzelm
tuned;
2019-08-06, by wenzelm
clarified modules: more direct data implementation;
2019-08-05, by wenzelm
Added Takeuchi function to HOL-ex
2019-08-06, by Manuel Eberl
full AFP test on lrzcloud2;
2019-08-05, by wenzelm
obsolete;
2019-08-05, by wenzelm
more efficient data structure;
2019-08-03, by wenzelm
clarified signature;
2019-08-03, by wenzelm
guard constraints by record_proofs=1, until performance implications have become more clear;
2019-08-03, by wenzelm
more complete completions according to Sorts.insert_complete_ars (cf. 13199740ced6), e.g. relevant for theories HOL-ex.Word_Type, HOL-Matrix_LP.SparseMatrix;
2019-08-03, by wenzelm
tuned;
2019-08-03, by wenzelm
tuned;
2019-08-03, by wenzelm
maintain sort constraints from type instantiations, with pro-forma derivation to collect oracles/thms;
2019-08-03, by wenzelm
more direct proofs for type classes;
2019-08-02, by wenzelm
tuned;
2019-08-02, by wenzelm
clarified modules: inference kernel maintains sort algebra within the logic;
2019-08-02, by wenzelm
more elementary treatment of standard_vars (unconstrainT is already standard);
2019-08-01, by wenzelm
clarified module structure;
2019-08-01, by wenzelm
simplified module structure: back to plain datatype (see 95f4f08f950f and 70019ab5e57f);
2019-08-01, by wenzelm
abstract type theory_id -- ensure non-equality type independently of implementation;
2019-08-01, by wenzelm
clarified export: retain proof boxes as local definitions -- more scalable;
2019-07-31, by wenzelm
reduced dependencies
2019-07-31, by nipkow
clarified global theory context;
2019-07-30, by wenzelm
more robust export, based on reconstruct_proof / expand_proof;
2019-07-30, by wenzelm
clarified modules: provide reconstruct_proof / expand_proof at the bottom of proof term construction;
2019-07-30, by wenzelm
tuned -- fewer warnings;
2019-07-30, by wenzelm
discontinued pointless messages;
2019-07-30, by wenzelm
clarified context;
2019-07-30, by wenzelm
clarified modules;
2019-07-30, by wenzelm
discontinue clean_proof: without type args its PThm nodes are not expanded, but with type args it is too unstable;
2019-07-30, by wenzelm
merged
2019-07-29, by wenzelm
more diagnostic operations;
2019-07-29, by wenzelm
tuned -- non-strict args;
2019-07-29, by wenzelm
proper constrains_map -- for shyps that are covered by present variables (amending 251f1fb44ccd);
2019-07-29, by wenzelm
tuned signature;
2019-07-29, by wenzelm
clarified signature;
2019-07-29, by wenzelm
tuned signature;
2019-07-29, by wenzelm
News for bind infixl
2019-07-29, by nipkow
Monadic bind is now infixl as is the norm
2019-07-29, by nipkow
purge remains from test (cf. 5a53724fe247);
2019-07-28, by wenzelm
tuned;
2019-07-28, by wenzelm
clarified signature;
2019-07-28, by wenzelm
removed obsolete RC tags;
2019-07-28, by wenzelm
tuned;
2019-07-28, by wenzelm
clarified signature;
2019-07-28, by wenzelm
tuned;
2019-07-28, by wenzelm
tuned;
2019-07-27, by wenzelm
clarified signature;
2019-07-27, by wenzelm
tuned;
2019-07-27, by wenzelm
tuned;
2019-07-27, by wenzelm
tuned;
2019-07-27, by wenzelm
tuned -- reorder sections;
2019-07-26, by wenzelm
tuned;
2019-07-26, by wenzelm
proper argument type (amending 42fbb6abed5a);
2019-07-26, by wenzelm
tuned signature;
2019-07-26, by wenzelm
tuned;
2019-07-26, by wenzelm
finalize proofs earlier to reduce memory requirement;
2019-07-26, by wenzelm
proper proof_serial;
2019-07-26, by wenzelm
more explicit type proof_serial;
2019-07-26, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
tip