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
+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.
simplified roundup activation interface;
2009-03-29, by wenzelm
merged
2009-03-28, by wenzelm
merged
2009-03-28, by haftmann
merged
2009-03-28, by haftmann
second attempt for code_deps command
2009-03-28, by haftmann
merged
2009-03-28, by haftmann
corrected projection of required statement names
2009-03-28, by haftmann
corrected check for additional type variables on rhs of code equations
2009-03-28, by haftmann
not yet fruitful tex experiments with bounding boxes
2009-03-28, by haftmann
simplified Locale.activate operations, using generic context;
2009-03-28, by wenzelm
renamed ProofContext.add_fixes_i to ProofContext.add_fixes, eliminated obsolete external version;
2009-03-28, by wenzelm
define_prefs: removed redundant Drule.gen_all, which is already part of the norm_hhf stage of Assumption.assume;
2009-03-28, by wenzelm
renamed ProofContext.note_thmss_i to ProofContext.note_thmss, eliminated obsolete external version;
2009-03-28, by wenzelm
simplified references to facts, eliminated external note_thmss;
2009-03-28, by wenzelm
added map_facts_refs;
2009-03-28, by wenzelm
tuned;
2009-03-28, by wenzelm
replaced add_binds(_i) by bind_terms -- internal version only;
2009-03-28, by wenzelm
replaced add_binds by singleton bind_term;
2009-03-28, by wenzelm
simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
2009-03-28, by wenzelm
minor tuning;
2009-03-28, by wenzelm
merged
2009-03-28, by wenzelm
Merged.
2009-03-28, by ballarin
Corrections to locale syntax.
2009-03-28, by ballarin
Update explanation of locale expressions to locale reimplementation.
2009-03-27, by ballarin
Comments updated.
2009-03-27, by ballarin
fixed proof
2009-03-27, by chaieb
merged
2009-03-27, by chaieb
fps made instance of number_ring
2009-03-27, by chaieb
updated keywords with polyml-experimental;
2009-03-27, by wenzelm
export position_of;
2009-03-27, by wenzelm
dropped infix union
2009-03-27, by haftmann
tuned notoriously slow metis proof
2009-03-27, by haftmann
merged
2009-03-27, by haftmann
dropped toy example Code_Antiq
2009-03-27, by haftmann
more convenient name uniqueness
2009-03-27, by haftmann
normalized imports
2009-03-27, by haftmann
dropped legacy goal package call
2009-03-27, by haftmann
merged
2009-03-27, by haftmann
merged
2009-03-26, by haftmann
step towards proper pictures in dvi
2009-03-26, by haftmann
merged
2009-03-26, by wenzelm
parameterize assoc_fold with is_numeral predicate
2009-03-26, by huffman
merged
2009-03-26, by paulson
New theorems mostly concerning infinite series.
2009-03-26, by paulson
interpretation/interpret: prefixes are mandatory by default;
2009-03-26, by wenzelm
interpretation/interpret: prefixes are mandatory by default;
2009-03-26, by wenzelm
interpretation/interpret: prefixes within locale expression are mandatory by default;
2009-03-26, by wenzelm
locale_expression: mandatory as parameter;
2009-03-26, by wenzelm
register_locale: produce stamps at the spot where elements are registered;
2009-03-26, by wenzelm
pretty_rule/print_results: no thm status here -- it is potentially slow and mostly uninformative/confusing as long as proofs are still unfinished;
2009-03-26, by wenzelm
pretty_thm_aux etc.: explicit show_status flag;
2009-03-26, by wenzelm
simplified attribute and method setup: eliminating bottom-up styles makes it easier to keep things in one place, and also SML/NJ happy;
2009-03-26, by wenzelm
@{binding} is not a constructor term and should not be inlined, otherwise we loose value polymorphism;
2009-03-25, by wenzelm
tuned;
2009-03-25, by wenzelm
use more informative Thm.proof_body_of for oracle demo;
2009-03-25, by wenzelm
Proofterm.approximate_proof_body;
2009-03-25, by wenzelm
fulfill_proof/thm_proof: pass whole proof_body, not just the projection to proof (which might be incomplete);
2009-03-25, by wenzelm
removed misleading make_proof_body, make_oracles, make_thms, which essentially assume a *full* proof;
2009-03-25, by wenzelm
avoid mixing of left/right associative infixes, to make it work with experimental Poly/ML 5.3 branch;
2009-03-25, by wenzelm
simplified addPrettyPrinter setup: may pass (fn ...) directly if type constraints are omitted -- addPrettyPrinter treated as a special case internally;
2009-03-24, by wenzelm
status_of: need to include local promises as well!
2009-03-24, by wenzelm
status_of: simultaneous list;
2009-03-24, by wenzelm
display derivation status of thms;
2009-03-24, by wenzelm
recover old ids;
2009-03-24, by wenzelm
report ML typing;
2009-03-24, by wenzelm
merged
2009-03-24, by wenzelm
merged
2009-03-24, by nipkow
NEWS: [arith]
2009-03-24, by nipkow
get_index: produce index of next pending token, not the last one;
2009-03-24, by wenzelm
register token positions persistently with context;
2009-03-24, by wenzelm
tuned;
2009-03-24, by wenzelm
more markup elements for ML programs;
2009-03-24, by wenzelm
merged
2009-03-24, by wenzelm
process at-sml-dev last -- takes very long (why?);
2009-03-24, by wenzelm
fix
2009-03-24, by nipkow
merged
2009-03-24, by nipkow
presburger uses [arith] now
2009-03-24, by nipkow
merged
2009-03-24, by wenzelm
merged
2009-03-24, by haftmann
added Imperative_HOL_ex
2009-03-24, by haftmann
Use assms rather than prems in find_theorems solves.
2009-03-24, by Timothy Bourke
clean up proofs of sign rules for multiplication; add list of lemmas mult_sign_intros
2009-03-23, by huffman
lemmas add_sign_intros
2009-03-23, by huffman
merged
2009-03-23, by haftmann
moved Imperative_HOL examples to Imperative_HOL/ex
2009-03-23, by haftmann
corrected variable renaming
2009-03-23, by haftmann
tuned error messages
2009-03-23, by haftmann
moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
2009-03-23, by haftmann
structure LinArith now named Lin_Arith
2009-03-23, by haftmann
suddenly infix identifier oo occurs in generated code
2009-03-23, by haftmann
datatype antiquote: maintain original Position.range, which is eventually attached to the resulting ML tokens;
2009-03-24, by wenzelm
eliminated non-canonical alias structure T = ML_Lex;
2009-03-24, by wenzelm
error "Static Errors";
2009-03-24, by wenzelm
more systematic type use_context;
2009-03-24, by wenzelm
tuned;
2009-03-23, by wenzelm
more systematic type use_context;
2009-03-23, by wenzelm
eliminated Output.ml_output;
2009-03-23, by wenzelm
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip