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.
merged
2012-09-19, by wenzelm
recording elapsed time in mutabelle for more detailed evaluation
2012-09-19, by bulwahn
Added missing predicators (for multisets and countable sets)
2012-09-18, by popescua
added top-level theory for Cardinals
2012-09-18, by popescua
group "simps" together
2012-09-18, by blanchet
register induct attributes
2012-09-18, by blanchet
further tuned simpset
2012-09-18, by blanchet
bnf_note_all mode for "pre_"-BNFs
2012-09-18, by traytel
separated registration of BNFs from bnf_def (BNFs are now stored only for bnf_def and (co)data commands)
2012-09-18, by traytel
tuned
2012-09-18, by nipkow
beautified names
2012-09-18, by nipkow
proved all upper bounds
2012-09-18, by nipkow
tuned simpset
2012-09-17, by blanchet
cleaner way of dealing with the set functions of sums and products
2012-09-17, by blanchet
handle the general case with more than two levels of nesting when discharging induction prem prems
2012-09-17, by blanchet
clean unfolding of prod and sum sets
2012-09-17, by blanchet
got rid of one "auto" in induction tactic
2012-09-17, by blanchet
cleaned up internal naming scheme for bnfs
2012-09-17, by traytel
more robust GUI component handlers;
2012-09-19, by wenzelm
more rendering;
2012-09-18, by wenzelm
minimal clipboard support (similar to org.lobobrowser.html.gui.HtmlBlockPanel);
2012-09-18, by wenzelm
output is read-only;
2012-09-18, by wenzelm
token marker for extended syntax styles;
2012-09-18, by wenzelm
pass base_snapshot to enable hyperlinks into other nodes;
2012-09-18, by wenzelm
more explicit message markup and rendering;
2012-09-18, by wenzelm
recover order of stacked markup;
2012-09-18, by wenzelm
some actual rich text markup via XML.content_markup;
2012-09-18, by wenzelm
proper separation of output messages;
2012-09-18, by wenzelm
some support for inital command markup;
2012-09-18, by wenzelm
more static rendering state;
2012-09-18, by wenzelm
Pretty_Text_Area is based on Rich_Text_Area;
2012-09-18, by wenzelm
renamed Text_Area_Painter to Rich_Text_Area;
2012-09-17, by wenzelm
tuned signature -- more general Text_Area_Painter operations;
2012-09-17, by wenzelm
tuned signature;
2012-09-17, by wenzelm
tuned signature;
2012-09-17, by wenzelm
tuned signature;
2012-09-17, by wenzelm
somewhat more general JEdit_Lib;
2012-09-17, by wenzelm
prefer official polyml-5.5.0;
2012-09-17, by wenzelm
bypass HOL-Mirabelle-ex in regular test, until its tendency to "hang" has been resolved;
2012-09-17, by wenzelm
merged
2012-09-17, by wenzelm
tuned
2012-09-17, by nipkow
updated to polyml-5.5.0;
2012-09-17, by wenzelm
some updates for polyml-5.5.0;
2012-09-17, by wenzelm
tuned
2012-09-17, by nipkow
alternative output panel, based on Pretty_Text_Area, based on JEditEmbeddedTextArea;
2012-09-16, by wenzelm
got rid of ad-hoc lift function
2012-09-16, by nipkow
converted wt into a set, tuned names
2012-09-16, by nipkow
use strip_typeN in bnf_def (instead of repairing strip_type)
2012-09-16, by traytel
removing find_theorems commands that were left in the developments accidently
2012-09-16, by bulwahn
tuning
2012-09-15, by blanchet
tuned code to avoid special case for "fun"
2012-09-15, by blanchet
tuned induction tactic
2012-09-15, by blanchet
tuned error message
2012-09-15, by blanchet
tuning
2012-09-15, by blanchet
typeclass formalising bounded subtraction
2012-09-15, by haftmann
dropped some unused identifiers
2012-09-15, by haftmann
export rel_mono theorem
2012-09-15, by traytel
merged two unfold steps
2012-09-14, by blanchet
took out one rotate_tac
2012-09-14, by blanchet
killed spurious rotate_tac; use auto instead of blast
2012-09-14, by blanchet
moved blast tactic to where it is actually needed
2012-09-14, by blanchet
fixed bug in "mk_map" for the "fun" case
2012-09-14, by blanchet
correct generalization to 3 or more mutually recursive datatypes
2012-09-14, by blanchet
provide more guidance, exploiting our knowledge of the goal
2012-09-14, by blanchet
fixed issue with bound variables in prem prems + tuning
2012-09-14, by blanchet
use right version of "mk_UnIN"
2012-09-14, by blanchet
select the right premise in "mk_induct_discharge_prem_prems_tac" instead of relying on backtracking
2012-09-14, by blanchet
tuned code before fixing "mk_induct_discharge_prem_prems_tac"
2012-09-14, by blanchet
tuned proofs;
2012-09-14, by wenzelm
merged
2012-09-14, by wenzelm
polished the induction
2012-09-14, by blanchet
put the flat at the right place (to avoid exceptions)
2012-09-14, by blanchet
fixed variable exporting problem
2012-09-14, by blanchet
compile
2012-09-14, by blanchet
added induct tactic
2012-09-14, by blanchet
tuning
2012-09-14, by blanchet
renamed "mk_UnN" to "mk_UnIN"
2012-09-14, by blanchet
merged two commands
2012-09-14, by blanchet
allow default values to refer to selector arguments -- this is useful, e.g. for tllist: ttl (TNil x) = TNil x (example by Andreas Lochbihler)
2012-09-14, by blanchet
distinguish between nested and nesting BNFs
2012-09-14, by blanchet
make tactic more robust in the case where "asm_simp_tac" already finishes the job
2012-09-14, by blanchet
derive induction via backward proof, to ensure that the premises are in the right order for constructors like "X x y x" where x and y are mutually recursive
2012-09-14, by blanchet
no longer react on global_settings (cf. 34ac36642a31);
2012-09-14, by wenzelm
refined output panel: more value-oriented approach to update and caret focus;
2012-09-14, by wenzelm
clarified markup names;
2012-09-14, by wenzelm
more general Document_Model.point_range;
2012-09-14, by wenzelm
more static handling of rendering options;
2012-09-14, by wenzelm
tuned options (again);
2012-09-14, by wenzelm
more scalable option-group;
2012-09-14, by wenzelm
tuned
2012-09-14, by nipkow
merged
2012-09-13, by wenzelm
tuned proofs;
2012-09-13, by wenzelm
remove theory Real_Integration, not needed since 44e42d392c6e when Euclidean spaces where introduced
2012-09-13, by hoelzl
workaround for HOL-Mirabelle-ex oddities;
2012-09-13, by wenzelm
instructions for quick start in 20min;
2012-09-13, by wenzelm
more liberal init_components: base dir may get created later when resolving missing components;
2012-09-13, by wenzelm
more efficient painting based on cached result;
2012-09-13, by wenzelm
more standard init_components -- particularly important to pick up correct jdk/scala version;
2012-09-13, by wenzelm
tuned
2012-09-13, by nipkow
merged
2012-09-12, by wenzelm
rough and ready induction
2012-09-12, by blanchet
nicer error message, indicating which type is empty (relying on metatheoretical completeness proof here)
2012-09-12, by blanchet
observe context more carefully when producing "fresh" variables -- for increased chances that method "subst" works in local context (including that of forked proofs);
2012-09-12, by wenzelm
eliminated some old material that is unused in the visible universe;
2012-09-12, by wenzelm
tuning
2012-09-12, by blanchet
set up things for (co)induction sugar
2012-09-12, by blanchet
tuning
2012-09-12, by blanchet
added sumEN_tupled_balanced
2012-09-12, by blanchet
load fonts into JavaFX as well;
2012-09-12, by wenzelm
some support for actual HTML rendering;
2012-09-12, by wenzelm
merged
2012-09-12, by wenzelm
free variable name tuning
2012-09-12, by blanchet
reuse generated names (they look better + slightly more efficient)
2012-09-12, by blanchet
desambiguate grammar (e.g. for Nil's mixfix ("[]"))
2012-09-12, by blanchet
avoided duplicate lemma
2012-09-12, by blanchet
put an underscore between names, for compatibility with old package (and also because it makes sense)
2012-09-12, by blanchet
got rid of metis calls
2012-09-12, by blanchet
tuning
2012-09-12, by blanchet
removed obsolete argument "int" and thus made SML/NJ happy (cf. 03bee3a6a1b7);
2012-09-12, by wenzelm
standardized ML aliases;
2012-09-12, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip