Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+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.
pretty_ml/ml_pretty: proper handling of markup and string length;
2009-03-23, by wenzelm
more systematic type use_context;
2009-03-23, by wenzelm
removed obsolete ml_output;
2009-03-23, by wenzelm
more systematic type use_context;
2009-03-23, by wenzelm
more systematic type use_context, with particular values ML_Parse.global_context and ML_Context.local_context;
2009-03-23, by wenzelm
de-camelized ML_Name_Space;
2009-03-23, by wenzelm
suppress status output for traditional tty modes (including Proof General);
2009-03-23, by wenzelm
added report_text -- status messages with text body;
2009-03-23, by wenzelm
maintain parse trees cumulatively;
2009-03-23, by wenzelm
Block markup: maintain output version within tree values (in accordance with String) -- changes operational behaviour wrt. print_mode;
2009-03-23, by wenzelm
future scheduler: reduced wait timeout if tasks need to be canceled -- to improve reactivity of interrupts;
2009-03-23, by wenzelm
merged
2009-03-23, by haftmann
Main is (Complex_Main) base entry point in library theories
2009-03-23, by haftmann
Main is (Complex_Main) base entry point in library theories
2009-03-23, by haftmann
added instances for bot, top, wellorder
2009-03-23, by haftmann
tuned header
2009-03-23, by haftmann
more canonical import, syntax fix
2009-03-23, by haftmann
merged
2009-03-23, by haftmann
merged
2009-03-22, by haftmann
more antiquotations
2009-03-22, by haftmann
moved import of module qelim to theory Presburger
2009-03-22, by haftmann
tuned header
2009-03-22, by haftmann
dropped theory Arith_Tools
2009-03-22, by haftmann
lemma nat_dvd_not_less moved here from Arith_Tools
2009-03-22, by haftmann
distributed contents of theory Arith_Tools to theories Int, IntDiv and NatBin accordingly
2009-03-22, by haftmann
merged
2009-03-22, by wenzelm
merged
2009-03-22, by nipkow
1. New cancellation simprocs for common factors in inequations
2009-03-22, by nipkow
clarified relationship of modules Code_Name and Code_Printer
2009-03-22, by haftmann
added Symreltab (binary relations of symbols) instance of TableFun
2009-03-22, by haftmann
proper signature;
2009-03-22, by wenzelm
added read_antiq, with improved error reporting;
2009-03-22, by wenzelm
ML_Lex.read_antiq;
2009-03-22, by wenzelm
ML_Lex.read_antiq;
2009-03-22, by wenzelm
simplified Antiquote.read (again);
2009-03-22, by wenzelm
export report -- version that actually covers all cases;
2009-03-22, by wenzelm
Test of advanced ML compiler invocation in Poly/ML 5.3.
2009-03-22, by wenzelm
ML/ml_test.ML: test of advanced ML compiler invocation in Poly/ML 5.3;
2009-03-22, by wenzelm
added pretty_ml;
2009-03-22, by wenzelm
export eval_antiquotes: refined version that operates on ML tokens;
2009-03-22, by wenzelm
ML_Lex.pos_of: regular position;
2009-03-22, by wenzelm
replaced Antiquote.is_antiq by Antiquote.is_text;
2009-03-22, by wenzelm
merged
2009-03-21, by wenzelm
extra toplevel pretty-printing for Poly/ML; experimental version for Poly/ML 5.3;
2009-03-21, by wenzelm
merged
2009-03-21, by wenzelm
merged
2009-03-21, by huffman
move field lemmas into class locale context
2009-03-21, by huffman
move diff_eq_0_iff_eq into class locale context
2009-03-21, by huffman
removed obsolete pprint operations;
2009-03-21, by wenzelm
added polyml_pp.ML: toplevel pretty printing for Poly/ML 4.x and 5.x before 5.3;
2009-03-21, by wenzelm
adapted toplevel_pp to ML_Pretty.pretty;
2009-03-21, by wenzelm
replaced install_pp/make_pp by more general toplevel_pp based on use_text;
2009-03-21, by wenzelm
simplified datatype ML_Pretty.pretty: model Isabelle not Poly/ML;
2009-03-21, by wenzelm
simplified datatype ML_Pretty.pretty: model Isabelle not Poly/ML;
2009-03-21, by wenzelm
Datatype for ML pretty printing (cf. mlsource/MLCompiler/Pretty.sml in Poly/ML 5.3).
2009-03-21, by wenzelm
Pretty.position;
2009-03-21, by wenzelm
added position;
2009-03-21, by wenzelm
added generic ML_Pretty interface;
2009-03-21, by wenzelm
restricted interrupts for tasks running as future worker thread -- attempt to prevent interrupt race conditions;
2009-03-21, by wenzelm
more ambitious ML_OPTIONS;
2009-03-21, by wenzelm
more stats;
2009-03-21, by wenzelm
added ML syntax markup;
2009-03-20, by wenzelm
report markup for ML tokens;
2009-03-20, by wenzelm
Antiquote.read: argument for reporting text;
2009-03-20, by wenzelm
future_job: do not inherit attributes, but enforce restricted interrupts -- attempt to prevent interrupt race conditions;
2009-03-20, by wenzelm
uniform ml_prompts for RAW and Pure;
2009-03-20, by wenzelm
eliminated old Addsimps;
2009-03-20, by wenzelm
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
2009-03-20, by wenzelm
fixed possibility_tac;
2009-03-20, by wenzelm
eliminated global SIMPSET, CLASET etc. -- refer to explicit context;
2009-03-20, by wenzelm
merged
2009-03-20, by wenzelm
merged
2009-03-20, by berghofe
split_codegen now eta-expands terms on-the-fly.
2009-03-20, by berghofe
proper context for prove_cont/adm_tac;
2009-03-20, by wenzelm
with_attributes: canonical capture/release scheme (potentially iron out race condition);
2009-03-20, by wenzelm
considerable speedup of benchmarks by using minimal simpset;
2009-03-20, by wenzelm
allow non-printable symbols within string tokens;
2009-03-20, by wenzelm
merged
2009-03-19, by wenzelm
add lemma det_diagonal; remove wellorder requirement on several lemmas
2009-03-19, by huffman
merged
2009-03-19, by haftmann
tuned some theorem and attribute bindings
2009-03-19, by haftmann
proper spacing before ML antiquotations -- note that @ may be part of symbolic ML identifiers;
2009-03-19, by wenzelm
eval_antiquotes: joint scanning of ML tokens and antiquotations;
2009-03-19, by wenzelm
added scan_antiq;
2009-03-19, by wenzelm
RAW: provide dummy Isar.main to make tty work gracefully (with ML toplevel);
2009-03-19, by wenzelm
added tokenize;
2009-03-19, by wenzelm
parameterized datatype antiquote and read operation;
2009-03-19, by wenzelm
Antiquote.Text: keep full position information;
2009-03-19, by wenzelm
OuterLex.read_antiq;
2009-03-19, by wenzelm
moved Isar/antiquote.ML to General/antiquote.ML, which is loaded early;
2009-03-19, by wenzelm
moved basic change_prompt, scan_string, scan_alt_string, scan_quoted to symbol_pos.ML;
2009-03-19, by wenzelm
use Name.of_binding for basic logical entities without name space (fixes, case names etc.);
2009-03-19, by wenzelm
Name.of_binding: proper full_name (with checks) before projecting base name;
2009-03-19, by wenzelm
merged
2009-03-19, by wenzelm
imported patch euclidean
2009-03-19, by huffman
Merged.
2009-03-18, by ballarin
Updated chapters 1-5 to locale reimplementation.
2009-03-18, by ballarin
command 'use', 'ML': apply ML environment to theory and target as well;
2009-03-19, by wenzelm
added map_contexts (cf. Proof.map_contexts);
2009-03-19, by wenzelm
tuned;
2009-03-19, by wenzelm
generalized ML_Context.inherit_env;
2009-03-18, by wenzelm
more precise type Symbol_Pos.text;
2009-03-18, by wenzelm
more precise type Symbol_Pos.text;
2009-03-18, by wenzelm
de-camelized Symbol_Pos;
2009-03-18, by wenzelm
Library.merge/OrdList.union: optimize the important special case where the tables coincide -- NOTE: this changes both the operational behaviour and the result for non-standard eq/ord notion;
2009-03-18, by wenzelm
reduced verbosity;
2009-03-18, by wenzelm
made SML/NJ happy
2009-03-18, by haftmann
tuned interpunctation
2009-03-18, by haftmann
strip_abss: always strip abstractions as far as possible, without keeping alternatives (which appear to be redundant anyway, but cause significant slowdown since discrimination nets collapse abstractions);
2009-03-17, by wenzelm
close/all_assm_tac: finish all subgoals from left to right (cf. Proof.goal_tac a28d83e903ce) -- NB: ALLGOALS/THEN_ALL_NEW operate from right to left;
2009-03-17, by wenzelm
reverted abbreviations: improved performance via Item_Net.T;
2009-03-17, by wenzelm
export match_rew -- useful for implementing "procs" for rewrite_term;
2009-03-17, by wenzelm
tuned comment;
2009-03-17, by wenzelm
merged
2009-03-17, by wenzelm
document new additions to HOL/Library
2009-03-16, by huffman
clean up proofs
2009-03-16, by huffman
adapted to general Item_Net;
2009-03-17, by wenzelm
turned structure NetRules into general Item_Net, which is loaded earlier;
2009-03-17, by wenzelm
renamed Tactic.taglist/untaglist/orderlist to tag_list/untag_list/order_list (in library.ML);
2009-03-17, by wenzelm
goal_tac: finish marked assumptions from left to right -- corresponds better with the strategy of etac, with significant performance gains in some situations;
2009-03-17, by wenzelm
eq_assumption: slightly more efficient by checking (open) result of Logic.assum_problems directly;
2009-03-17, by wenzelm
tuned aeconv: test plain aconv before expensive eta_contract;
2009-03-17, by wenzelm
substantial speedup of assumption and elim-resolution: Logic.assum_problems refrains from eager application of parameters, discriminate via Term.could_unify before invoking full unification (assumes terms in beta-normal form, as do higher term net operations anyway);
2009-03-16, by wenzelm
refined is_norm_hhf: reject beta-redexes (rules based on term nets or could_unify assume normal form), also potentially faster by avoiding expensive Envir.beta_eta_contract;
2009-03-16, by wenzelm
provide Simplifier.norm_hhf(_protect) as regular simplifier operation;
2009-03-16, by wenzelm
method parser: pass proper context;
2009-03-16, by wenzelm
merged
2009-03-16, by wenzelm
simplified method setup;
2009-03-16, by wenzelm
updated generated file;
2009-03-16, by wenzelm
simplifief 'method_setup' command;
2009-03-16, by wenzelm
spelling;
2009-03-16, by wenzelm
export method parser;
2009-03-16, by wenzelm
adapted 'method_setup' command to Method.setup;
2009-03-16, by wenzelm
tuned signature;
2009-03-16, by wenzelm
have remote script interrupted like the other provers
2009-03-16, by immler
simplified method setup;
2009-03-15, by wenzelm
export section, sections;
2009-03-15, by wenzelm
merged
2009-03-15, by wenzelm
updated NEWS
2009-03-14, by immler
use goal instead of Proof State
2009-03-14, by immler
split relevance-filter and writing of problem-files;
2009-03-14, by immler
show certain errors to the user
2009-03-14, by immler
removed connection check;
2009-03-14, by immler
merged
2009-03-15, by wenzelm
merged
2009-03-14, by haftmann
reverted to old version of Set.thy -- strange effects have to be traced first
2009-03-14, by haftmann
simplified attribute and method setup;
2009-03-15, by wenzelm
simplified attribute setup;
2009-03-15, by wenzelm
simplified attribute setup;
2009-03-15, by wenzelm
updated generated files;
2009-03-15, by wenzelm
added 'attribute_setup' command;
2009-03-15, by wenzelm
added setup and attribute_setup -- expect plain parser instead of syntax function;
2009-03-15, by wenzelm
ML_Syntax.make_binding;
2009-03-15, by wenzelm
added make_binding;
2009-03-15, by wenzelm
removed obsolete no_base_names naming policy;
2009-03-14, by wenzelm
merged
2009-03-13, by wenzelm
merged
2009-03-13, by haftmann
coherent binding policy with primitive target operations
2009-03-13, by haftmann
moved some generic nonsense to arith_data.ML
2009-03-13, by haftmann
tuned ML code
2009-03-13, by haftmann
remove legacy ML bindings
2009-03-13, by huffman
simplified method setup;
2009-03-13, by wenzelm
simplified goal_spec: default to first goal;
2009-03-13, by wenzelm
eliminated type Args.T;
2009-03-13, by wenzelm
added simplified setup;
2009-03-13, by wenzelm
pervasive types 'a parser and 'a context_parser;
2009-03-13, by wenzelm
unified type Proof.method and pervasive METHOD combinators;
2009-03-13, by wenzelm
more regular method setup via SIMPLE_METHOD;
2009-03-13, by wenzelm
tuned Method exports: non-pervasive type method (cf. Proof.method), pervasive METHOD combinators;
2009-03-13, by wenzelm
merged
2009-03-13, by wenzelm
fix typed print translation for CARD('a)
2009-03-13, by huffman
introduce new helper functions; clean up proofs
2009-03-13, by huffman
merged
2009-03-13, by nipkow
added comment
2009-03-13, by nipkow
hiding numeric coercions in LaTeX
2009-03-13, by nipkow
merged
2009-03-13, by haftmann
dropped spurious `quote` tags
2009-03-13, by haftmann
merged
2009-03-12, by haftmann
tuned
2009-03-12, by haftmann
strippd Id
2009-03-12, by haftmann
vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
2009-03-12, by haftmann
tuned
2009-03-12, by haftmann
consider exit status of code generation direcitve
2009-03-12, by haftmann
provide regular ML interfaces for Isar source language elements;
2009-03-13, by wenzelm
get data from plain Proof.context;
2009-03-13, by wenzelm
more user aliases;
2009-03-12, by wenzelm
merged
2009-03-12, by wenzelm
remove trailing spaces
2009-03-12, by huffman
remove trailing spaces
2009-03-12, by huffman
simplified preparation and outer parsing of specification;
2009-03-12, by wenzelm
simplified preparation and outer parsing of specification;
2009-03-12, by wenzelm
removed legacy_infer_term, legacy_infer_prop;
2009-03-12, by wenzelm
old name_spec for 'axioms' and 'defs' (from spec_parse.ML);
2009-03-12, by wenzelm
added legacy type inference (from fixrec_package.ML);
2009-03-12, by wenzelm
simplified versions check_spec, read_spec, check_free_spec, read_free_spec: operate on list of singleton statements;
2009-03-12, by wenzelm
removed old named_spec, spec_name, spec_opt_name;
2009-03-12, by wenzelm
keep dead code fresh;
2009-03-12, by wenzelm
tuned;
2009-03-12, by wenzelm
merged
2009-03-12, by wenzelm
merged
2009-03-12, by nipkow
added div lemmas
2009-03-12, by nipkow
merged
2009-03-12, by nipkow
optional latex sugar
2009-03-12, by nipkow
Assumption.all_prems_of, Assumption.all_assms_of;
2009-03-12, by wenzelm
Assumption.local_prems_of;
2009-03-12, by wenzelm
renamed assms_of to all_assms_of, and prems_of to all_prems_of;
2009-03-12, by wenzelm
axiomatization: more precise treatment of binding;
2009-03-12, by wenzelm
renamed sticky_prefix to mandatory_path;
2009-03-12, by wenzelm
replaced old-style add_path/no_base_names by sticky_prefix;
2009-03-12, by wenzelm
updated according to actual manual title;
2009-03-12, by wenzelm
renamed NameSpace.bind to NameSpace.define;
2009-03-12, by wenzelm
renamed bind to define;
2009-03-12, by wenzelm
tuned signature;
2009-03-12, by wenzelm
updated generated files;
2009-03-12, by wenzelm
tuned;
2009-03-12, by wenzelm
added 'local_setup' command;
2009-03-11, by wenzelm
debugging: special handling of EXCURSION_FAIL;
2009-03-11, by wenzelm
tuned;
2009-03-11, by wenzelm
delete unused generated files;
2009-03-11, by wenzelm
basic setup for "main" as generated Isabelle manual;
2009-03-11, by wenzelm
tuned;
2009-03-11, by wenzelm
merged
2009-03-11, by wenzelm
merged
2009-03-11, by haftmann
fixed typo
2009-03-11, by haftmann
(restored previous version)
2009-03-11, by haftmann
corrected type inference of primitive definitions
2009-03-11, by haftmann
HOLogic.mk_set, HOLogic.dest_set
2009-03-11, by haftmann
tuned
2009-03-11, by haftmann
tuned funny error message
2009-03-11, by haftmann
stripped dead code
2009-03-11, by haftmann
min_weak_def [code del]
2009-03-11, by haftmann
renamed (unused?) "split.splits" to split_splits -- it was only accepted by accident;
2009-03-11, by wenzelm
merged
2009-03-11, by wenzelm
Extended approximation boundaries by fractions and base-2 floating point numbers
2009-03-11, by hoelzl
Added "What's in Main" to doc sources
2009-03-11, by nipkow
merged
2009-03-11, by nipkow
Docs
2009-03-11, by nipkow
Updated paths in Decision_Procs comments and NEWS
2009-03-11, by hoelzl
eliminated qualified_names naming policy: qualified names are only permitted via explicit Binding.qualify/qualified_name etc. (NB: user-level outer syntax should never do this);
2009-03-11, by wenzelm
more precise treatment of qualified bindings;
2009-03-11, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip