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.
inter and union are mere abbreviations for inf and sup
2009-09-19, by haftmann
merged
2009-09-24, by haftmann
lemma relating fold1 and foldl; code_unfold rules for Inf_fin, Sup_fin, Min, Max, Inf, Sup
2009-09-24, by haftmann
subsumed by more general setup in List.thy
2009-09-24, by haftmann
idempotency case for fold1
2009-09-24, by haftmann
added dual for complete lattice
2009-09-24, by haftmann
merged
2009-09-24, by nipkow
record how many "proof"s are solved by s/h
2009-09-24, by nipkow
added quotes for filenames;
2009-09-24, by boehmes
merged; adopted to changes from Code_Evaluation in the predicate compiler
2009-09-24, by bulwahn
replaced sorry by oops; removed old debug functions in predicate compiler
2009-09-23, by bulwahn
added first version of quickcheck based on the predicate compiler; added a few quickcheck examples
2009-09-23, by bulwahn
adapted configuration for DatatypeCase.make_case
2009-09-23, by bulwahn
added a new example for the predicate compiler
2009-09-23, by bulwahn
added context free grammar example; removed dead code; adapted to work without quick and dirty mode; fixed typo
2009-09-23, by bulwahn
added first prototype of the extended predicate compiler
2009-09-23, by bulwahn
moved predicate compiler to Tools
2009-09-23, by bulwahn
removed generation of strange tuple modes in predicate compiler
2009-09-23, by bulwahn
extending predicate compiler and proof procedure to support tuples; testing predicate wirh HOL-MicroJava semantics
2009-09-23, by bulwahn
modified predicate compiler further to support tuples
2009-09-23, by bulwahn
changed preprocessing due to problems with LightweightJava; added transfer of thereoms; changed the type of mode to support tuples in the predicate compiler
2009-09-23, by bulwahn
handling of definitions
2009-09-23, by bulwahn
experimenting to add some useful interface for definitions
2009-09-23, by bulwahn
added predicate compile preprocessing structure for definitional thms -- probably is replaced by hooking the theorem command differently
2009-09-23, by bulwahn
modified handling of side conditions in proof procedure of predicate compiler
2009-09-23, by bulwahn
merged
2009-09-23, by haftmann
Code_Eval(uation)
2009-09-23, by haftmann
merged
2009-09-23, by blanchet
Added "nitpick_const_simp" tags to lazy list theories.
2009-09-23, by blanchet
atbroy101 is long dead, use atbroy99; comment out broken SML test invocation
2009-09-23, by krauss
merged
2009-09-23, by haftmann
stripped legacy ML bindings
2009-09-23, by haftmann
Undo errornous commit of Statespace change
2009-09-23, by hoelzl
correct variable order in approximate-method
2009-09-23, by hoelzl
merged
2009-09-23, by paulson
Correct chasing of type variable instantiations during type unification.
2009-09-23, by paulson
hide newly introduced constants
2009-09-23, by haftmann
used standard fold function and type aliases
2009-09-22, by Philipp Meyer
sos method generates and uses proof certificates
2009-09-21, by Philipp Meyer
full reserve of worker threads -- for improved CPU utilization;
2009-09-22, by wenzelm
merged
2009-09-22, by haftmann
be more cautious wrt. simp rules: inf_absorb1, inf_absorb2, sup_absorb1, sup_absorb2 are no simp rules by default any longer
2009-09-22, by haftmann
tail -n 20: more helpful output if make fails
2009-09-22, by krauss
corrected order of type variables in code equations; more precise certificate for cases
2009-09-22, by haftmann
merged
2009-09-21, by Christian Urban
tuned some proofs
2009-09-21, by Christian Urban
merged
2009-09-21, by haftmann
added session theory for Bali and Nominal_Examples
2009-09-21, by haftmann
added session theory for Nominal_Examples
2009-09-21, by haftmann
added session theory for Bali
2009-09-21, by haftmann
adjusted to new Number Theory scenario
2009-09-21, by haftmann
added session entry point theories
2009-09-21, by haftmann
common base for protocols with symmetric keys
2009-09-21, by haftmann
tuned header
2009-09-21, by haftmann
isarified proof
2009-09-21, by haftmann
fixed permissions -- this is a script, not an executable;
2009-09-21, by wenzelm
tuned;
2009-09-21, by wenzelm
deleted unused file
2009-09-21, by boehmes
merged
2009-09-21, by haftmann
entry point theory for examples; reactivated half-dead example
2009-09-21, by haftmann
merged
2009-09-21, by boehmes
corrected remote SMT solver invocation
2009-09-21, by boehmes
theory entry point for session Hoare_Parallel (now also with proper underscore)
2009-09-21, by haftmann
merged
2009-09-21, by boehmes
tuned author
2009-09-21, by boehmes
added new method "smt": an oracle-based connection to external SMT solvers
2009-09-18, by boehmes
tuned tracing;
2009-09-20, by wenzelm
scheduler backdoor: 9999 means 1 worker;
2009-09-20, by wenzelm
Hilbert_Classical: more precise control of parallel_proofs;
2009-09-20, by wenzelm
actually observe Multithreading.enabled (cf. d302f1c9e356);
2009-09-20, by wenzelm
merged
2009-09-19, by nipkow
restructured code
2009-09-19, by nipkow
merged
2009-09-19, by haftmann
rewrite premises in tactical proof also with inf_fun_eq and inf_bool_eq: attempt to allow user to use inf [=>] and inf [bool] in his specs
2009-09-18, by haftmann
modified minimization log
2009-09-18, by nipkow
merged
2009-09-18, by nipkow
skip &&& goals
2009-09-18, by nipkow
INTER and UNION are mere abbreviations for INFI and SUPR
2009-09-18, by haftmann
simplified proof
2009-09-18, by haftmann
partially isarified proof
2009-09-18, by haftmann
tuned const_name antiquotations
2009-09-18, by haftmann
more antiquotations
2009-09-18, by haftmann
be more cautious wrt. simp rules: sup1_iff, sup2_iff, inf1_iff, inf2_iff, SUP1_iff, SUP2_iff, INF1_iff, INF2_iff are no longer simp by default
2009-09-18, by haftmann
tuned NEWS, added CONTRIBUTORS
2009-09-18, by haftmann
merged
2009-09-17, by nipkow
removed misleading log line
2009-09-17, by nipkow
NEWS: New method metisFT
2009-09-17, by paulson
New theorems for proving equalities and inclusions involving unions
2009-09-17, by paulson
added time limit for extraction phase (not supported on Cygwin)
2009-09-17, by boehmes
merged
2009-09-17, by boehmes
undo changes from revision 719426c9e1eb: removed Perl script for ATP invocation, measuring time using Bash-builtin "time";
2009-09-17, by boehmes
Synchronized.value does not require locking, since assigments are atomic;
2009-09-16, by wenzelm
tuned;
2009-09-16, by wenzelm
replaced opaque signature matching by plain old abstype (again, cf. ac4498f95d1c) -- this recovers pretty printing in SML/NJ and Poly/ML 5.3;
2009-09-16, by wenzelm
merged
2009-09-16, by haftmann
Inter and Union are mere abbreviations for Inf and Sup; tuned
2009-09-16, by haftmann
Inter and Union are mere abbreviations for Inf and Sup
2009-09-16, by haftmann
merged
2009-09-16, by nipkow
revised lemma counting
2009-09-16, by nipkow
merged
2009-09-16, by haftmann
merged
2009-09-15, by haftmann
hide new constants
2009-09-15, by haftmann
merged
2009-09-15, by haftmann
restored code generation for OCaml
2009-09-15, by haftmann
added singleton example
2009-09-15, by haftmann
added emptiness check predicate and singleton projection
2009-09-15, by haftmann
added append_after (tuned version of former insert_after of Seq);
2009-09-16, by wenzelm
double linking for improved performance of "prev";
2009-09-15, by wenzelm
merged
2009-09-15, by wenzelm
added hard timeout for sledgehammer based on elapsed time (no need to trust ATP's timeout handling);
2009-09-15, by boehmes
Isar.define_command: identify transaction;
2009-09-15, by wenzelm
updated bib;
2009-09-15, by wenzelm
count number of iterations required for minimization (and fixed bug: minimization was always called)
2009-09-14, by nipkow
merged
2009-09-14, by haftmann
more antiquotations
2009-09-14, by haftmann
some lemmas about strict order in lattices
2009-09-14, by haftmann
explicitly export type abbreviations (as usual in SML97);
2009-09-13, by wenzelm
wrapper for Real.fmt -- via StringCvt.realfmt;
2009-09-13, by wenzelm
made SML/NJ happy;
2009-09-13, by wenzelm
standard headers and text sections;
2009-09-12, by wenzelm
merged
2009-09-11, by nipkow
Made record parameter flexible to allow for extensions
2009-09-11, by nipkow
merged
2009-09-11, by haftmann
corrected upper/lowercase
2009-09-11, by haftmann
merged
2009-09-10, by haftmann
obey underscore naming convention
2009-09-10, by haftmann
plain structure name; signature constraint; shorter lines
2009-09-10, by haftmann
split of test examples from NatTransfer
2009-09-10, by haftmann
generic transfer procedure
2009-09-10, by haftmann
early bootstrap of generic transfer procedure
2009-09-10, by haftmann
cleanedup theorems all_nat ex_nat
2009-09-10, by haftmann
atp_minimize is now not using whitelist
2009-09-10, by Philipp Meyer
position information is now passed to all actions;
2009-09-10, by nipkow
logging number of metis lemmas
2009-09-10, by nipkow
minimization: comparing w/ and w/o.
2009-09-09, by nipkow
merged
2009-09-09, by haftmann
dropped accidental code additions
2009-09-09, by haftmann
merged
2009-09-09, by haftmann
explicit transfer avoids spurious merge problems
2009-09-09, by haftmann
moved eq handling in nbe into separate oracle
2009-09-09, by haftmann
tuned document -- proper text instead of source comments, reduced line length;
2009-09-08, by wenzelm
fixed cleanup routine in neos csdp script
2009-09-01, by Philipp Meyer
timeout option for ATPs
2009-09-08, by boehmes
merged
2009-09-07, by wenzelm
modernized Event_Bus -- based on actors;
2009-09-07, by wenzelm
Fixed "minimal" to cover the case that "p []" holds (excluded in the article by Bradley & Manna)
2009-09-07, by nipkow
merged
2009-09-07, by nipkow
tuned stats
2009-09-07, by nipkow
Fixed a few problems with the method metisFT
2009-09-07, by paulson
merged
2009-09-07, by nipkow
tuned stats
2009-09-07, by nipkow
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
2009-09-07, by paulson
merged
2009-09-07, by paulson
conflict resolution possibly
2009-09-07, by paulson
New method, metisFT: a fully-typed proof search that should eliminate type errors during reconstruction
2009-09-04, by paulson
merged
2009-08-28, by paulson
More streamlining using metis.
2009-08-27, by paulson
enabled metis permanently, tuned stats
2009-09-07, by nipkow
added signature ATP_MINIMAL,
2009-09-05, by boehmes
merged
2009-09-05, by boehmes
separate output of ATP user time and sledgehammer (ML code) user time
2009-09-05, by boehmes
Mirabelle: command-line action options may either be key=value or just key
2009-09-05, by boehmes
added initialization and cleanup of actions,
2009-09-05, by boehmes
merged
2009-09-04, by haftmann
tuned metis proofs
2009-09-04, by haftmann
tuned
2009-09-04, by boehmes
tuned output
2009-09-04, by nipkow
merged
2009-09-03, by boehmes
Mirabelle: actions are responsible for catching exceptions and producing suitable log messages (makes log message uniform),
2009-09-03, by boehmes
merged
2009-09-03, by haftmann
merged
2009-09-03, by haftmann
proper class syntax for sublocale class < expr
2009-09-03, by haftmann
added option full_typed for sledgehammer action
2009-09-03, by boehmes
added runtime information to sledgehammer
2009-09-03, by boehmes
tuned
2009-09-03, by boehmes
scaled avg_time
2009-09-03, by nipkow
merged
2009-09-03, by nipkow
tuned
2009-09-03, by nipkow
isatest: collect test results and logs in testdata repository
2009-09-03, by krauss
replaced backlist by whitelist
2009-09-03, by boehmes
Mirabelle: logging of exceptions (works only for PolyML)
2009-09-03, by boehmes
merged
2009-09-02, by wenzelm
refined delay into delay_first/delay_last;
2009-09-02, by wenzelm
merged
2009-09-02, by boehmes
add report script for Mirabelle
2009-09-02, by boehmes
Mirabelle: actions are responsible for handling exceptions,
2009-09-02, by boehmes
removed errors overseen in previous changes
2009-09-02, by boehmes
moved Mirabelle from HOL/Tools to HOL,
2009-09-02, by boehmes
removed unused signature
2009-09-02, by boehmes
explicit checks;
2009-09-02, by wenzelm
updated Poly/ML SVN version;
2009-09-02, by wenzelm
eval/location_props: always produce YXML markup, independent of print_mode;
2009-09-02, by wenzelm
reorganized Compute theories for HOL-Matrix -- avoiding theory files within main HOL/Tools;
2009-09-02, by wenzelm
tuned ML message;
2009-09-02, by wenzelm
added "using" to blacklist
2009-09-02, by nipkow
merged
2009-09-02, by wenzelm
merged
2009-09-02, by wenzelm
removed old Isar document model;
2009-09-01, by wenzelm
corrected spelling
2009-09-01, by haftmann
merged
2009-09-01, by haftmann
added -q switch for run in qnd mode
2009-09-01, by haftmann
code generator is now a separate component
2009-09-01, by haftmann
tuned document
2009-09-01, by haftmann
some reorganization of number theory
2009-09-01, by haftmann
some reorganization of number theory
2009-09-01, by haftmann
merged
2009-09-01, by haftmann
tuned
2009-09-01, by haftmann
avoid long line
2009-08-24, by haftmann
added txt to blacklist
2009-09-01, by nipkow
Isabelle_Process: receiver as Actor, not EventBus;
2009-09-01, by wenzelm
merged
2009-09-01, by boehmes
Mirabelle: actions are responsible for their log messages, output is better readable
2009-09-01, by boehmes
merged
2009-09-01, by wenzelm
merged
2009-09-01, by boehmes
Mirabelle: added preliminary documentation,
2009-09-01, by boehmes
Mirabelle: explicit command blacklist, preliminary documentation
2009-08-31, by boehmes
modernized Isar_Document;
2009-09-01, by wenzelm
modernized Thy_Header;
2009-09-01, by wenzelm
misc cleanup and internal reorganization;
2009-09-01, by wenzelm
added linear_set.scala from http://isabelle.in.tum.de/repos/isabelle-jedit/rev/d567692f9717
2009-09-01, by wenzelm
moved lemma Wellfounded.in_inv_image to Relation.thy
2009-08-31, by krauss
moved wfrec to Recdef.thy
2009-08-31, by krauss
no consts_code for wfrec, as it violates the "code generation = equational reasoning" principle
2009-08-31, by krauss
Mirabelle: handle possible parser exceptions, emit suitable log message
2009-08-31, by boehmes
merged
2009-08-31, by boehmes
sledgehammer's temporary files are removed properly (even in case of an exception occurs)
2009-08-31, by boehmes
merged
2009-08-31, by nipkow
tuned the simp rules for Int involving insert and intervals.
2009-08-31, by nipkow
Mirabelle sledgehammer: added option to keep problem files, enabled "metis" switch again (was accidentally removed)
2009-08-31, by boehmes
Mirabelle: proper parsing of theorem names found by sledgehammer, respecting test intervals given along with file names
2009-08-31, by boehmes
merged
2009-08-29, by boehmes
apply metis with found theorems in case sledgehammer was successful
2009-08-29, by boehmes
propagate theorem names, in addition to generated return message
2009-08-29, by boehmes
misc tuning;
2009-08-29, by wenzelm
eliminated hard tabs;
2009-08-29, by wenzelm
moved Pure/Tools/isabelle_syntax.scala to Pure/System/isabelle_syntax.scala;
2009-08-29, by wenzelm
merged
2009-08-28, by wenzelm
fixed HOLogic.stringT
2009-08-28, by krauss
merged
2009-08-28, by nipkow
tuned proofs
2009-08-28, by nipkow
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip