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.
retain literal non-HHF assumptions, to facilitate re-import in Generic_Target.import_export_proof;
2012-04-03, by wenzelm
another attempt to avoid duplication of global vs. local syntax (reminiscent of old fork_mixfix);
2012-04-03, by wenzelm
export into target context (again), to retain its 'defines' (e.g. abbreviation lcoeff in theory HOL/Algebra/UnivPoly);
2012-04-03, by wenzelm
better drop background syntax if entity depends on parameters;
2012-04-03, by wenzelm
more uniform abbrev vs. define;
2012-04-03, by wenzelm
tuned;
2012-04-03, by wenzelm
clarified generic_const vs. close_schematic_term;
2012-04-03, by wenzelm
tuned;
2012-04-03, by wenzelm
more uniform theory_abbrev with const_declaration;
2012-04-03, by wenzelm
avoid const_declaration in aux. context (cf. locale_foundation);
2012-04-03, by wenzelm
clarified background_foundation vs. theory_foundation (with const_declaration);
2012-04-03, by wenzelm
tuned;
2012-04-03, by wenzelm
more general standard_declaration;
2012-04-02, by wenzelm
better restore after close_target;
2012-04-02, by wenzelm
tuned;
2012-04-02, by wenzelm
clarified standard_declaration vs. theory_declaration;
2012-04-02, by wenzelm
smarter generic_const: plain alias for non-dependent case (e.g. prospective datatype or record syntax);
2012-04-02, by wenzelm
tuned;
2012-04-02, by wenzelm
tuned;
2012-04-02, by wenzelm
tuned signature;
2012-04-02, by wenzelm
misc tuning and simplification;
2012-04-02, by wenzelm
better restore to first target, not last target;
2012-04-02, by wenzelm
refined define/abbrev: allow extra fixes in aux. context vs. bottom target (NB: export_term expands defined variables, leaving fixed ones);
2012-04-02, by wenzelm
more general Local_Theory.restore, allow any nesting level;
2012-04-02, by wenzelm
new tutorial
2012-04-02, by nipkow
New manual Programming and Proving in Isabelle/HOL
2012-04-02, by nipkow
add simp rules for dvd on negative numerals
2012-04-02, by huffman
merged, manually resolving conflicts due to session renaming (cf. 6488c5efec49)
2012-04-01, by krauss
clarified terminology; added reference to bundle component
2012-04-01, by krauss
less modest NEWS; CONTRIBUTORS
2012-04-01, by krauss
renamed import session back to Import, conforming to directory name; NEWS
2012-04-01, by krauss
more precise IsaMakefile (eg. see HOL-Algebra);
2012-04-01, by wenzelm
more keywords;
2012-04-01, by wenzelm
merged
2012-04-01, by wenzelm
merged
2012-04-01, by krauss
removed old HOL4 import -- corresponding exporter is lost, code is broken, no users known, maintenance nightmare
2012-04-01, by krauss
Modernized HOL-Import for HOL Light
2012-04-01, by Cezary Kaliszyk
merged
2012-04-01, by wenzelm
adapted Mira configuration to dd04c8173bb2.
2012-04-01, by krauss
removed Nat_Numeral.thy, moving all theorems elsewhere
2012-04-01, by huffman
less brutal return from function, to allow caller to report error;
2012-04-01, by wenzelm
more general context command with auxiliary fixes/assumes etc.;
2012-04-01, by wenzelm
more precise type annotation (cf. 6523a21076a8);
2012-04-01, by wenzelm
nothing specific about named target;
2012-04-01, by wenzelm
clarified Generic_Target.notes: always perform Attrib.partial_evaluation;
2012-04-01, by wenzelm
added Attrib.global_notes/local_notes/generic_notes convenience;
2012-04-01, by wenzelm
simplified;
2012-04-01, by wenzelm
tuned signature;
2012-04-01, by wenzelm
clarified Named_Target.target_declaration: propagate through other levels as well;
2012-04-01, by wenzelm
Local_Theory.map_contexts with explicit level indication: 0 = main target at bottom;
2012-04-01, by wenzelm
tuned proofs
2012-04-01, by huffman
merged
2012-03-31, by huffman
tuned proof
2012-03-31, by huffman
add lemma power_le_one
2012-03-31, by huffman
tuned;
2012-03-31, by wenzelm
tuned signature;
2012-03-31, by wenzelm
more direct Local_Defs.contract;
2012-03-31, by wenzelm
more precise Local_Defs.expand wrt. *local* prems only;
2012-03-31, by wenzelm
tuned comment;
2012-03-31, by wenzelm
more robust Scala 2.9.x interpreter invocation -- avoid separate interpreter thread and thus deadlock of Swing_Thread.now;
2012-03-30, by wenzelm
tuned;
2012-03-30, by wenzelm
dropped empty files
2012-03-30, by haftmann
dropped now obsolete Cset theories
2012-03-30, by haftmann
merged
2012-03-30, by wenzelm
tuned proofs, less guesswork;
2012-03-30, by wenzelm
merged
2012-03-30, by huffman
load Tools/numeral.ML in Num.thy
2012-03-30, by huffman
tuned proof
2012-03-30, by huffman
set up numeral reorient simproc in Num.thy
2012-03-30, by huffman
remove redundant simp rule
2012-03-30, by huffman
add simp rules for eve/odd on numerals
2012-03-30, by huffman
remove content-free theory ex/Arithmetic_Series_Complex.thy
2012-03-30, by huffman
rephrase lemmas about arithmetic series using numeral '2'
2012-03-30, by huffman
rephrase lemma card_Pow using '2' instead of 'Suc (Suc 0)'
2012-03-30, by huffman
replace lemmas eval_nat_numeral with a simpler reformulation
2012-03-30, by huffman
restate various simp rules for word operations using pred_numeral
2012-03-30, by huffman
new lemmas for simplifying subtraction on nat numerals
2012-03-30, by huffman
removed redundant nat-specific copies of theorems
2012-03-30, by huffman
move more theorems from Nat_Numeral.thy to Num.thy
2012-03-30, by huffman
"invariant" is free in main HOL (cf. 56adbf5bcc82, e64ffc96a49f);
2012-03-30, by wenzelm
more robust ISABELLE_JDK_HOME settings, based on exisiting JAVA_HOME provided by isatest shell environment (which depends a lot on the host);
2012-03-30, by wenzelm
more explicit isatest environment settings (from private .bashrc);
2012-03-30, by wenzelm
merged
2012-03-30, by huffman
fix search-and-replace errors
2012-03-30, by huffman
move lemma card_UNIV_bool from Nat_Numeral.thy to Finite_Set.thy
2012-03-30, by huffman
add constant pred_numeral k = numeral k - (1::nat);
2012-03-30, by huffman
move lemmas from Nat_Numeral.thy to Nat.thy
2012-03-30, by huffman
move lemmas from Nat_Numeral to Int.thy and Num.thy
2012-03-30, by huffman
merged
2012-03-30, by bulwahn
adding theory to prove completeness of the exhaustive generators
2012-03-30, by bulwahn
refine bindings in quickcheck_common: do not conceal and do not declare as simps
2012-03-30, by bulwahn
hiding fact not so aggressively
2012-03-30, by bulwahn
power on predicate relations
2012-03-30, by haftmann
made Mirabelle-SH's 'trivial' check optional;
2012-03-30, by sultana
merged
2012-03-29, by wenzelm
more specific notion of partiality (cf. Scala version);
2012-03-29, by wenzelm
use qualified names for rsp and rep_eq theorems in quotient_def
2012-03-29, by kuncar
announcing NEWS (cf. 446cfc760ccf)
2012-03-29, by bulwahn
remove obsolete simp rule for powers
2012-03-29, by huffman
remove duplicate lemmas power_m1_{even,odd} in favor of power_minus1_{even,odd}
2012-03-29, by huffman
remove unneeded rewrite rules for powers of numerals
2012-03-29, by huffman
remove duplicate lemma Suc_numeral
2012-03-29, by huffman
move many lemmas from Nat_Numeral.thy to Power.thy or Num.thy
2012-03-29, by huffman
bootstrap Num.thy before Power.thy;
2012-03-29, by huffman
educated guess to include jdk
2012-03-29, by haftmann
improved robustness with new antiquoation by Makarius
2012-03-28, by nipkow
merged
2012-03-28, by nipkow
updates
2012-03-28, by nipkow
updated documentation files (cf. c14fda8fee38)
2012-03-28, by bulwahn
clarified ISABELLE_JDK_HOME: derive from running JVM, but ignore accidental JAVA_HOME;
2012-03-28, by wenzelm
merged
2012-03-28, by wenzelm
removed references to obsolete theorems
2012-03-28, by huffman
merged
2012-03-28, by bulwahn
some tuning while reviewing the current state of the quotient_def package
2012-03-28, by bulwahn
improving spelling
2012-03-28, by bulwahn
changing more definitions to quotient_definition
2012-03-28, by bulwahn
removing now redundant impl_of theorems in DAList
2012-03-28, by bulwahn
using abstract code equations for proofs of code equations in Multiset
2012-03-28, by bulwahn
simplified statements and proofs;
2012-03-28, by wenzelm
tuned whitespace;
2012-03-28, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip