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.
options as first argument to check functions
2010-10-25, by bulwahn
changing test parameters in examples to get to a result within the global timelimit
2010-10-25, by bulwahn
adding a global fixed timeout to quickcheck
2010-10-25, by bulwahn
adding a global time limit to the values command
2010-10-25, by bulwahn
explicit message_output thread, with flushing after timeout, ensure atomic user-operations without the danger of IO Interrupt;
2010-10-25, by wenzelm
more explicit indication of Output.Private_Hooks (still public to accomodate clones of Proof General for now);
2010-10-25, by wenzelm
renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
2010-10-25, by wenzelm
explicitly qualify type Output.output, which is a slightly odd internal feature;
2010-10-25, by wenzelm
export main ML entry by default;
2010-10-25, by wenzelm
observe Isabelle/ML coding standards;
2010-10-25, by wenzelm
merged
2010-10-25, by wenzelm
significantly improved Isabelle/Isar implementation manual;
2010-10-25, by wenzelm
misc tuning;
2010-10-25, by wenzelm
removed some remains of Output.debug (follow-up to fce2202892c4);
2010-10-25, by wenzelm
recovered some odd two-dimensional layout;
2010-10-25, by wenzelm
merged
2010-10-25, by haftmann
dropped (almost) redundant distinct.induct rule; distinct_simps again named distinct.simps
2010-10-25, by haftmann
moved sledgehammer to Plain; tuned dependencies
2010-10-25, by haftmann
CONTRIBUTORS
2010-10-25, by haftmann
merge
2010-10-25, by blanchet
merged
2010-10-25, by blanchet
updated keywords
2010-10-25, by blanchet
introduced manual version of "Auto Solve" as "solve_direct"
2010-10-25, by blanchet
make "sledgehammer_params" work on single-threaded platforms
2010-10-25, by blanchet
tuning
2010-10-22, by blanchet
handle timeouts (to prevent failure from other threads);
2010-10-22, by blanchet
update keywords
2010-10-25, by haftmann
some partial_function examples
2010-10-25, by krauss
added ML antiquotation @{assert};
2010-10-25, by wenzelm
updated keywords;
2010-10-25, by wenzelm
integrated partial_function into HOL-Plain
2010-10-23, by krauss
first version of partial_function package
2010-10-23, by krauss
Complete_Partial_Order.thy: complete partial orders over arbitrary chains, with fixpoint theorem
2010-10-23, by krauss
merged
2010-10-25, by bulwahn
splitting Hotel Key card example into specification and the two tests for counter example generation
2010-10-22, by bulwahn
adding generator quickcheck
2010-10-22, by bulwahn
restructuring values command and adding generator compilation
2010-10-22, by bulwahn
moving general functions from core_data to predicate_compile_aux
2010-10-22, by bulwahn
updating to new notation in commented examples
2010-10-22, by bulwahn
merged
2010-10-24, by huffman
use default names sprod/Rep_sprod/Abs_sprod from pcpodef instead of Sprod/Rep_Sprod/Abs_Sprod; similarly for ssum
2010-10-24, by huffman
remove legacy comp_dbind option from domain package
2010-10-23, by huffman
change fixrec parser to not accept theorem names with (unchecked) option
2010-10-23, by huffman
tuned
2010-10-23, by huffman
rename lemma surjective_pairing_Sprod2 to spair_sfst_ssnd
2010-10-22, by huffman
add lemma strict3
2010-10-22, by huffman
do proofs using Rep_Sprod_simps, Rep_Ssum_simps; remove unused lemmas
2010-10-22, by huffman
make discrete_cpo a subclass of chfin; remove chfin instances for fun, cfun
2010-10-22, by huffman
direct instantiation unit :: discrete_cpo
2010-10-22, by huffman
remove finite_po class
2010-10-22, by huffman
simplify proofs about flift; remove unneeded lemmas
2010-10-22, by huffman
simplify proof
2010-10-22, by huffman
minimize imports
2010-10-21, by huffman
add type annotation to avoid warning
2010-10-21, by huffman
simplify some proofs, convert to Isar style
2010-10-21, by huffman
rename lemma spair_lemma to spair_Sprod
2010-10-21, by huffman
pcpodef (open) 'a lift
2010-10-21, by huffman
remove intro! attribute from {sinl,sinr}_defined
2010-10-21, by huffman
simplify proofs of ssumE, sprodE
2010-10-21, by huffman
merged
2010-10-24, by wenzelm
renamed nat_number
2010-10-24, by nipkow
nat_number -> eval_nat_numeral
2010-10-24, by nipkow
some cleanup in Function_Lib
2010-10-22, by krauss
merged
2010-10-22, by blanchet
compile
2010-10-22, by blanchet
added SMT solver to Sledgehammer docs
2010-10-22, by blanchet
more robust handling of "remote_" vs. non-"remote_" provers
2010-10-22, by blanchet
generalized the relevance filter so that it takes the list of "irrelevant constants" as argument (since the ATP and SMT preprocessing are different)
2010-10-22, by blanchet
replaced references with proper record that's threaded through
2010-10-22, by blanchet
fixed signature of "is_smt_solver_installed";
2010-10-22, by blanchet
renamed modules
2010-10-22, by blanchet
renamed files
2010-10-22, by blanchet
took out "smt"/"remote_smt" from default ATPs until they are properly implemented
2010-10-22, by blanchet
remove more needless code ("run_smt_solvers");
2010-10-22, by blanchet
got rid of duplicate functionality ("run_smt_solver_somehow");
2010-10-22, by blanchet
bring ATPs and SMT solvers more in line with each other
2010-10-22, by blanchet
make Sledgehammer minimizer fully work with SMT
2010-10-22, by blanchet
generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well
2010-10-22, by blanchet
first step in adding support for an SMT backend to Sledgehammer
2010-10-21, by blanchet
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
2010-10-21, by blanchet
cosmetics
2010-10-21, by blanchet
relation method: re-check given term with type constraints to avoid unspecific failure if ill-typed -- keep old behaviour for tactic version
2010-10-22, by krauss
Changed section title to please LaTeX.
2010-10-22, by hoelzl
temporary removed Predicate_Compile_Quickcheck_Examples from tests
2010-10-21, by bulwahn
adapting alternative_defs, predicate_compile_quickcheck, examples and code_prolog
2010-10-21, by bulwahn
using a signature in core_data and moving some more functions to core_data
2010-10-21, by bulwahn
splitting large core file into core_data, mode_inference and predicate_compile_proof
2010-10-21, by bulwahn
added generator_dseq compilation for a sound depth-limited compilation with small value generators
2010-10-21, by bulwahn
for now safely but unpractically assume no predicate is terminating
2010-10-21, by bulwahn
adding decreasing bind and non-decreasing bind; depth-limited and depth-unlimited compilation possible
2010-10-21, by bulwahn
adding option smart_depth_limiting to predicate compiler
2010-10-21, by bulwahn
merged
2010-10-20, by huffman
introduce function strict :: 'a -> 'b -> 'b, which works like Haskell's seq; use strict instead of strictify in various definitions
2010-10-20, by huffman
add lemma lub_eq_bottom_iff
2010-10-20, by huffman
combine check_and_sort_domain with main function; rewrite much of the error-checking code
2010-10-20, by huffman
constructor arguments with selectors must have pointed types
2010-10-20, by huffman
simplify check_and_sort_domain; more meaningful variable names
2010-10-20, by huffman
replace fixrec 'permissive' mode with per-equation 'unchecked' option
2010-10-19, by huffman
rename domain_theorems.ML to domain_induction.ML; rename domain_extender.ML to domain.ML
2010-10-19, by huffman
simplify some proofs; remove some unused lists of lemmas
2010-10-19, by huffman
replace 'in_defl' relation and '_ ::: _' syntax with 'defl_set' function
2010-10-19, by huffman
eliminate constant 'coerce'; use 'prj oo emb' instead
2010-10-19, by huffman
simplify fixrec pattern match function
2010-10-19, by huffman
simplify some proofs
2010-10-17, by huffman
tuned
2010-10-19, by Christian Urban
added some facts about factorial and dvd, div and mod
2010-10-19, by bulwahn
removing something that probably slipped into the Quotient_List theory
2010-10-19, by bulwahn
Quotient package: partial equivalence introduction
2010-10-19, by Cezary Kaliszyk
reorganisation of the FSet theory (changed the primary naming scheme of constants and theorems to *_fset)
2010-10-18, by Christian Urban
remove dead code
2010-10-16, by huffman
remove old uses of 'simp_tac HOLCF_ss'
2010-10-16, by huffman
merged
2010-10-16, by huffman
remove last few dependencies on domain_library.ML and delete it; temporarily disable emptiness check
2010-10-16, by huffman
reimplement proof automation for coinduct rules
2010-10-16, by huffman
add functions mk_imp, mk_all
2010-10-16, by huffman
move emptiness check to comp_theorems; remove eqs parameter to prove_induction; remove dead code
2010-10-15, by huffman
simplify automation of induct proof
2010-10-15, by huffman
add function mk_adm
2010-10-15, by huffman
rewrite proof automation for finite_ind; get rid of case_UU_tac
2010-10-15, by huffman
put constructor argument specs in constr_info type
2010-10-14, by huffman
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip