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.
layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
2010-05-12, by boehmes
integrated SMT into the HOL image
2010-05-12, by boehmes
replaced More_conv.top_conv (which does not re-apply the given conversion to its results, only to the result's subterms) by Simplifier.full_rewrite
2010-05-12, by boehmes
use proper context operations (for fresh names of type and term variables, and for hypothetical definitions), monomorphize theorems (instead of terms, necessary for hypothetical definitions made during lambda lifting)
2010-05-12, by boehmes
split monolithic Z3 proof reconstruction structure into separate structures, use one set of schematic theorems for all uncertain proof rules (to extend proof reconstruction by missing cases), added several schematic theorems, improved abstraction of goals (abstract all uninterpreted sub-terms, only leave builtin symbols)
2010-05-12, by boehmes
added tracing of reconstruction data
2010-05-12, by boehmes
added new SMT translation files which use a simpler intermediate term representation and a simpler translation of builtin symbols, have less overhead for renaming symbols and generating the signature, add come with a simpler separation of formulas and terms
2010-05-12, by boehmes
deleted SMT translation files (to be replaced by a simplified version)
2010-05-12, by boehmes
move the addition of extra facts into a separate module
2010-05-12, by boehmes
normalize numerals: also rewrite Numeral0 into 0
2010-05-12, by boehmes
added missing rewrite rules for natural min and max
2010-05-12, by boehmes
rewrite bool case expressions as if expression
2010-05-12, by boehmes
simplified normalize_rule and moved it further down in the code
2010-05-12, by boehmes
merged addition of rules into one function
2010-05-12, by boehmes
added simplification for distinctness of small lists
2010-05-12, by boehmes
moved the addition of DLO tactic into the Z3 theory (DLO is required only for Z3 proof reconstruction)
2010-05-12, by boehmes
added Proofterm.unconstrain_thm_proof for Thm.unconstrainT -- loosely based on the version by krauss/schropp;
2010-05-14, by wenzelm
conditionally unconstrain thm proofs -- loosely based on the version by krauss/schropp;
2010-05-13, by wenzelm
the_classrel/the_arity: avoid Thm.transfer for proofterm version -- theory might already have become stale within the proof_body future;
2010-05-13, by wenzelm
avoid redundant rebinding of name/prop -- probably introduced accidentally in 80bb72a0f577;
2010-05-13, by wenzelm
raise Fail uniformly for proofterm errors, which appear to be rather low-level;
2010-05-13, by wenzelm
unconstrainT operations on proofs, according to krauss/schropp;
2010-05-13, by wenzelm
added Proofterm.get_name variants according to krauss/schropp;
2010-05-13, by wenzelm
conditional structure SingleAssignment;
2010-05-12, by wenzelm
merged
2010-05-12, by wenzelm
merged
2010-05-12, by haftmann
tuned proofs and fact and class names
2010-05-12, by haftmann
tuned fact collection names and some proofs
2010-05-12, by haftmann
grouped local statements
2010-05-12, by haftmann
tuned test problems
2010-05-12, by haftmann
merged
2010-05-12, by wenzelm
merged
2010-05-12, by nipkow
simplified proof
2010-05-12, by nipkow
modernized specifications;
2010-05-12, by wenzelm
updated/unified some legacy warnings;
2010-05-12, by wenzelm
tuned;
2010-05-12, by wenzelm
do not emit legacy_feature warnings here -- users have no chance to disable them;
2010-05-12, by wenzelm
removed obsolete CVS Ids;
2010-05-12, by wenzelm
removed some obsolete admin stuff;
2010-05-12, by wenzelm
check NEWS;
2010-05-12, by wenzelm
removed obsolete CVS Ids;
2010-05-12, by wenzelm
updated some version numbers;
2010-05-12, by wenzelm
minor tuning;
2010-05-12, by wenzelm
reverted parts of 7902dc7ea11d -- note that NEWS of published Isabelle releases are essentially read-only;
2010-05-12, by wenzelm
merged
2010-05-12, by wenzelm
merged
2010-05-12, by haftmann
modernized specifications; tuned reification
2010-05-12, by haftmann
merged
2010-05-12, by haftmann
added lemmas concerning last, butlast, insort
2010-05-12, by haftmann
Remove RANGE_WARN
2010-05-12, by Cezary Kaliszyk
clarified NEWS entry
2010-05-12, by hoelzl
merged
2010-05-12, by hoelzl
added NEWS entry
2010-05-12, by hoelzl
Added atLeastAtMost_singleton_iff, atLeastAtMost_singleton'
2010-05-11, by hoelzl
Add rules directly to the corresponding class locales instead.
2010-05-11, by hoelzl
Removed usage of normalizating locales.
2010-05-11, by hoelzl
speed up some proofs, fixing linarith_split_limit warnings
2010-05-11, by huffman
fix some linarith_split_limit warnings
2010-05-11, by huffman
include iszero_simps in semiring_norm just once (they are already included in rel_simps)
2010-05-11, by huffman
fix duplicate simp rule warning
2010-05-11, by huffman
no more RealPow.thy (remaining lemmas moved to RealDef.thy)
2010-05-11, by huffman
merged
2010-05-11, by huffman
simplify code for emptiness check
2010-05-11, by huffman
removed lemma real_sq_order; use power2_le_imp_le instead
2010-05-11, by huffman
merged
2010-05-11, by haftmann
merged
2010-05-11, by haftmann
represent de-Bruin indices simply by position in list
2010-05-11, by haftmann
tuned reification functions
2010-05-11, by haftmann
tuned code; toward a tightended interface with generated code
2010-05-11, by haftmann
fix spelling of 'superseded'
2010-05-11, by huffman
NEWS: removed theory PReal
2010-05-11, by huffman
collected NEWS updates for HOLCF
2010-05-11, by huffman
merged
2010-05-11, by huffman
move floor lemmas from RealPow.thy to RComplete.thy
2010-05-11, by huffman
add lemma tendsto_Complex
2010-05-11, by huffman
move some theorems from RealPow.thy to Transcendental.thy
2010-05-11, by huffman
add lemma power2_eq_1_iff; generalize some other lemmas
2010-05-11, by huffman
minimize imports
2010-05-10, by huffman
move lemma real_mult_is_one to Rings.thy, renamed to square_eq_1_iff
2010-05-10, by huffman
clarified Pretty.font_metrics;
2010-05-12, by wenzelm
format as topmost list of "divs", not just adjacent "spans" -- for proper line breaking;
2010-05-12, by wenzelm
tuned;
2010-05-12, by wenzelm
more precise pretty printing based on actual font metrics;
2010-05-11, by wenzelm
predefined spaces;
2010-05-11, by wenzelm
merged
2010-05-11, by wenzelm
support Isabelle plugin properties with defaults;
2010-05-11, by wenzelm
merged
2010-05-11, by Christian Urban
tuned proof so that no simplifier warning is printed
2010-05-11, by Christian Urban
renamed former Int.int_induct to Int.int_of_nat_induct, former Presburger.int_induct to Int.int_induct: is more conservative and more natural than the intermediate solution
2010-05-11, by haftmann
merged
2010-05-11, by haftmann
tuned
2010-05-11, by haftmann
theorem Presburger.int_induct has been renamed to Int.int_bidirectional_induct
2010-05-11, by haftmann
tuned; dropped strange myassoc2
2010-05-10, by haftmann
stylized COOPER exception
2010-05-10, by haftmann
simplified oracle
2010-05-10, by haftmann
shorten names
2010-05-10, by haftmann
updated references to ML files
2010-05-10, by haftmann
only one module fpr presburger method
2010-05-10, by haftmann
moved int induction lemma to theory Int as int_bidirectional_induct
2010-05-10, by haftmann
tuned theory text; dropped unused lemma
2010-05-10, by haftmann
one structure is better than three
2010-05-10, by haftmann
less complex organization of cooper source code
2010-05-10, by haftmann
dropped unused bindings; avoid open (documents dependency on generated code more explicitly)
2010-05-10, by haftmann
add real_mult_commute to legacy theorem names
2010-05-10, by huffman
new construction of real numbers using Cauchy sequences
2010-05-10, by huffman
add more credits to ex/Dedekind_Real.thy
2010-05-10, by huffman
put construction of reals using Dedekind cuts in HOL/ex
2010-05-10, by huffman
disable two stage save by default, to avoid change of file permissions (notably the dreaded executable bit on Cygwin);
2010-05-11, by wenzelm
simple dialogs: ensure Swing thread;
2010-05-10, by wenzelm
font size re-adjustment according to Lobo internals;
2010-05-10, by wenzelm
Scala for Netbeans 6.8v1.1.0rc2;
2010-05-10, by wenzelm
more convenient get_font;
2010-05-10, by wenzelm
renamed Config.get_thy to Config.get_global etc. to indicate that this is not the real thing;
2010-05-10, by wenzelm
more convenient look-and-feel setup;
2010-05-10, by wenzelm
more convenient get_font;
2010-05-10, by wenzelm
explicit getLines(n) ensures platform-independence -- our files follow the POSIX standard, not DOS;
2010-05-10, by wenzelm
updated to jedit 4.3.2;
2010-05-10, by wenzelm
ignore spurious TIMEOUT messages, maybe caused by change of actor semantics in scala-2.8;
2010-05-10, by wenzelm
adapted to scala-2.8.0.RC2;
2010-05-10, by wenzelm
merged
2010-05-10, by wenzelm
real_mult_commute -> mult_commute
2010-05-09, by huffman
avoid using real-specific versions of generic lemmas
2010-05-09, by huffman
avoid using real-specific versions of generic lemmas
2010-05-09, by huffman
remove a couple of redundant lemmas; simplify some proofs
2010-05-09, by huffman
merged
2010-05-09, by huffman
add lemmas one_less_inverse and one_le_inverse
2010-05-08, by huffman
do not redeclare [simp] rules, to avoid "duplicate rewrite rule" warnings
2010-05-09, by krauss
added lemmas rel_comp_UNION_distrib(2)
2010-05-09, by krauss
made SML/NJ happy;
2010-05-08, by wenzelm
reactivated Thm.legacy_unconstrainT for Nbe.lift_triv_classes_conv;
2010-05-09, by wenzelm
Thm.unconstrainT based on Logic.unconstrainT -- no proofterm yet;
2010-05-09, by wenzelm
just one version of Thm.unconstrainT, which affects all variables;
2010-05-09, by wenzelm
added Logic.unconstrain_allTs, based on calculations_for_thm_proof by krauss/schropp, but treat type variables uniformly as in strip_shyps (in thm.ML) or stripped_sorts (in more_thm.ML);
2010-05-09, by wenzelm
tuned;
2010-05-09, by wenzelm
removed unused "option" variants of "same" operations;
2010-05-09, by wenzelm
more basic replacement of newlines;
2010-05-09, by wenzelm
static Symbol.spaces;
2010-05-09, by wenzelm
proper use of var stopped;
2010-05-08, by wenzelm
removed junk;
2010-05-08, by wenzelm
tuned headers;
2010-05-08, by wenzelm
tuned;
2010-05-08, by wenzelm
merged
2010-05-08, by wenzelm
merged
2010-05-08, by haftmann
moved normalization proof tool infrastructure to canonical algebraic classes
2010-05-08, by haftmann
added lemmas
2010-05-08, by nipkow
merged
2010-05-08, by haftmann
renamed Normalizer to the more specific Semiring_Normalizer
2010-05-07, by haftmann
delete Groebner_Basis directory -- only one file left
2010-05-07, by haftmann
split of semiring normalization from Groebner theory; moved field_comp_conv to Numeral_Simproces
2010-05-07, by haftmann
merged
2010-05-07, by haftmann
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip