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.
moved lemma zdvd_period to theory Int
2010-05-07, by haftmann
tuned;
2010-05-08, by wenzelm
discontinued Pretty.setdepth, which appears to be largely unused, but can disrupt important markup if enabled accidentally;
2010-05-08, by wenzelm
tuned error message: regular Pretty.string_of instead of raw Pretty.output;
2010-05-08, by wenzelm
unified/simplified Pretty.margin_default;
2010-05-08, by wenzelm
renamed Thm.get_name -> Thm.derivation_name and Thm.put_name -> Thm.name_derivation, to emphasize the true nature of these operations;
2010-05-08, by wenzelm
prefer Thm.get_name_hint, which is closer to a user-space idea of "theorem name";
2010-05-08, by wenzelm
tuned signature;
2010-05-08, by wenzelm
added of_sort_proof according to krauss/schropp, with slightly more direct canonical_instance;
2010-05-08, by wenzelm
back-patching of axclass proofs;
2010-05-08, by wenzelm
back-patching via Single_Assignment.var;
2010-05-08, by wenzelm
support several sidekick parsers -- very basic default parser;
2010-05-07, by wenzelm
sidekick: unformatted content, notably without newlines;
2010-05-07, by wenzelm
unformatted output;
2010-05-07, by wenzelm
output symbolic pretty printing markup and format in the front end;
2010-05-07, by wenzelm
Pretty.formatted operates directly on XML trees, treating XML.Elem like a pro-forma block of indentation 0, like the ML version;
2010-05-07, by wenzelm
tuned;
2010-05-07, by wenzelm
strip_shyps_proof: dummy TFrees are called "'dummy" as in del_conflicting_tvars below;
2010-05-07, by wenzelm
use existing undefined function;
2010-05-07, by wenzelm
merged
2010-05-07, by wenzelm
removed semicolons
2010-05-07, by krauss
rule subrelI (for nice Isar proofs of relation inequalities)
2010-05-07, by krauss
merged
2010-05-07, by wenzelm
merged
2010-05-07, by haftmann
prefix normalizing replaces class_semiring
2010-05-07, by haftmann
xsymbolized
2010-05-06, by haftmann
moved method syntax here
2010-05-06, by haftmann
tuned proof
2010-05-06, by haftmann
former free-floating field_comp_conv now in structure Normalizer
2010-05-06, by haftmann
proper sublocales; no free-floating ML sections
2010-05-06, by haftmann
moved some lemmas from Groebner_Basis here
2010-05-06, by haftmann
revert to loose merge semantics
2010-05-06, by haftmann
merged
2010-05-06, by haftmann
moved generic lemmas to appropriate places
2010-05-06, by haftmann
tuned
2010-05-06, by haftmann
dropped duplicate comp_arith
2010-05-06, by haftmann
avoid open; tuned references to theorems
2010-05-06, by haftmann
avoid references to groebner bases in names which have no references to groebner bases
2010-05-06, by haftmann
tuned whitespace
2010-05-06, by haftmann
tuned headings
2010-05-06, by haftmann
avoid open
2010-05-06, by haftmann
tuned internal structure
2010-05-06, by haftmann
fail on merge of conflicting normalization entries: functions are not mergable
2010-05-06, by haftmann
more canonical data administration
2010-05-06, by haftmann
removed former algebra presimpset entirely
2010-05-06, by haftmann
removed former algebra presimpset from accessor
2010-05-06, by haftmann
removed former algebra presimpset from signature
2010-05-06, by haftmann
moved presimplification rules for algebraic methods into named thms functor
2010-05-06, by haftmann
tuned whitespace; dropped superfluous open
2010-05-06, by haftmann
dropped auxiliary method sring_norm; integrated normalizer.ML and normalizer_data.ML
2010-05-06, by haftmann
moved nat_arith ot Nat_Numeral: clarified normalizer setup
2010-05-05, by haftmann
dropped unused file
2010-05-05, by haftmann
dropped Id
2010-05-05, by haftmann
remove unused constant preal_of_rat; remove several unused lemmas about preals
2010-05-06, by huffman
respectfullness and preservation of prod_rel
2010-05-06, by Cezary Kaliszyk
ProofContext.init_global
2010-05-06, by haftmann
merged
2010-05-06, by haftmann
farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
2010-05-05, by haftmann
constant name access lattice is not in use any longer
2010-05-06, by haftmann
uniform treatment of length = 1 for forced breaks, also makes ML/Pretty.length coincide with Scala/XML.content_length;
2010-05-06, by wenzelm
replaced slightly odd fbreak markup by plain "\n", which also coincides with regular linebreaks produced outside the ML pretty engine;
2010-05-06, by wenzelm
added separate;
2010-05-06, by wenzelm
basic formatting of pretty trees;
2010-05-06, by wenzelm
added content_length;
2010-05-06, by wenzelm
slightly more general Library.chunks;
2010-05-06, by wenzelm
misc tuning -- accumulate body via ListBuffer;
2010-05-06, by wenzelm
basic support for symbolic pretty printing;
2010-05-06, by wenzelm
extractors for document updates;
2010-05-06, by wenzelm
extractors for outer keyword declarations;
2010-05-06, by wenzelm
eliminated deprecated "--" method;
2010-05-05, by wenzelm
use IndexedSeq instead of deprecated RandomAccessSeq, which is merely an alias;
2010-05-05, by wenzelm
use SwingApplication instead of deprecated GUIApplication;
2010-05-05, by wenzelm
simplified via Position extractors;
2010-05-05, by wenzelm
some rearrangement of Scala sources;
2010-05-05, by wenzelm
fminus and some more theorems ported from Finite_Set.
2010-05-05, by Cezary Kaliszyk
eq_morphism is always optional: avoid trivial morphism for empty list of equations
2010-05-05, by haftmann
tuned whitespace
2010-05-05, by haftmann
tuned interpunctation, dropped dead comment
2010-05-05, by haftmann
merged
2010-05-04, by huffman
avoid using '...' with LIMSEQ (cf. 1cc4ab4b7ff7)
2010-05-04, by huffman
generalize some lemmas to class t1_space
2010-05-04, by huffman
simplify definition of t1_space; generalize lemma closed_sing and related lemmas
2010-05-04, by huffman
generalize some lemmas
2010-05-04, by huffman
convert comments to 'text' blocks
2010-05-04, by huffman
generalize more lemmas about limits
2010-05-04, by huffman
repaired comments where SOMEthing went utterly wrong (cf. 2b04504fcb69)
2010-05-05, by krauss
merged
2010-05-04, by huffman
generalize types of LIMSEQ and LIM; generalize many lemmas
2010-05-04, by huffman
make (f -- a --> x) an abbreviation for (f ---> x) (at a)
2010-05-04, by huffman
make (X ----> L) an abbreviation for (X ---> L) sequentially
2010-05-04, by huffman
adapt to removed premise on tendsto lemma (cf. 88f0125c3bd2)
2010-05-04, by huffman
declare cont_discrete_cpo [cont2cont]
2010-05-04, by huffman
remove unneeded constant Zseq
2010-05-03, by huffman
add lemmas eventually_nhds_metric and tendsto_mono
2010-05-03, by huffman
remove unneeded premise
2010-05-03, by huffman
add constants netmap and nhds
2010-05-03, by huffman
Merged.
2010-05-04, by ballarin
Provide internal function for printing a single interpretation.
2010-05-04, by ballarin
Explicitly manage export in dependencies.
2010-04-27, by ballarin
fixed proof (cf. edc381bf7200);
2010-05-04, by wenzelm
Corrected imports; better approximation of dependencies.
2010-05-04, by hoelzl
Add Convex to Library build
2010-05-04, by hoelzl
Removed unnecessary assumption
2010-05-04, by hoelzl
Translating lemmas from Finite_Set to FSet.
2010-05-04, by Cezary Kaliszyk
merged
2010-05-04, by wenzelm
merged
2010-05-04, by berghofe
Turned Sem into an inductive definition.
2010-05-04, by berghofe
Corrected handling of "for" parameters.
2010-05-04, by berghofe
induct_true_def and induct_false_def are already contained in induct_rulify_fallback.
2010-05-04, by berghofe
added lemma about irreflexivity of pointer inequality in Imperative_HOL
2010-05-04, by bulwahn
added function ffilter and some lemmas from Finite_Set to the FSet theory
2010-05-04, by bulwahn
merged
2010-05-04, by haftmann
avoid if on rhs of default simp rules
2010-05-04, by haftmann
avoid exception Empty on malformed goal
2010-05-04, by krauss
locale predicates of classes carry a mandatory "class" prefix
2010-05-04, by haftmann
a ring_div is a ring_1_no_zero_divisors
2010-05-04, by haftmann
NEWS
2010-05-04, by haftmann
merged
2010-05-03, by huffman
merged
2010-05-01, by huffman
complete_lattice instance for net type
2010-05-01, by huffman
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip