Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+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
2010-10-29, by wenzelm
added user aliasses (still unclear how to specify names with whitespace contained)
2010-10-29, by haftmann
merged
2010-10-29, by haftmann
tuned structure of theory
2010-10-29, by haftmann
remove term_of equations for Heap type explicitly
2010-10-29, by haftmann
no need for setting up the kodkodi environment since Kodkodi 1.2.9
2010-10-29, by blanchet
fixed order of quantifier instantiation in new Skolemizer
2010-10-29, by blanchet
restructure Skolemization code slightly
2010-10-29, by blanchet
ensure that MESON correctly preserves the name of variables (needed by the new Skolemizer)
2010-10-29, by blanchet
more work on new Skolemizer without Hilbert_Choice
2010-10-29, by blanchet
fix cluster numbering in the absense of Hilbert_Choice (reverts acde1b606b0e, effectively reintroducing most of 0bfaaa81fc62)
2010-10-29, by blanchet
prevent type errors because of inconsistent skolem Var types by giving fresh indices to Skolems
2010-10-29, by blanchet
make handling of parameters more robust, by querying the goal
2010-10-29, by blanchet
actually pass "verbose" argument
2010-10-29, by haftmann
eliminated obsolete \_ escape;
2010-10-29, by wenzelm
eliminated obsolete \_ escapes in rail environments;
2010-10-29, by wenzelm
proper markup of formal text;
2010-10-29, by wenzelm
merged
2010-10-29, by wenzelm
hide_const various constants, in particular to avoid ugly qualifiers in HOLCF
2010-10-29, by krauss
reverted e31e3f0071d4 because "foo.bar(5)" (with quotes) is wrong
2010-10-29, by blanchet
merged
2010-10-29, by Lars Noschinski
Remove unnecessary premise of mult1_union
2010-09-22, by Lars Noschinski
adapting HOL-Mutabelle to changes in quickcheck
2010-10-29, by bulwahn
NEWS
2010-10-29, by bulwahn
changed global fixed timeout to a configurable timeout for quickcheck; test parameters in quickcheck are now fully passed around with the context
2010-10-29, by bulwahn
updating documentation on quickcheck in the Isar reference
2010-10-29, by bulwahn
merged
2010-10-28, by bulwahn
adding a simple check to only run with a SWI-Prolog version known to work
2010-10-28, by bulwahn
tuned messages;
2010-10-28, by wenzelm
discontinued obsolete ML antiquotation @{theory_ref};
2010-10-28, by wenzelm
tuned;
2010-10-28, by wenzelm
moved FOL/ex/Iff_Oracle.thy to HOL/ex where it is more accessible to most readers of isar-ref;
2010-10-28, by wenzelm
type attribute is derived concept outside the kernel;
2010-10-28, by wenzelm
preserve original source position of exn;
2010-10-28, by wenzelm
handle Type.TYPE_MATCH, not arbitrary exceptions via MATCH_TYPE variable;
2010-10-28, by wenzelm
use Exn.interruptible_capture to keep user-code interruptible (Exn.capture not immediately followed by Exn.release here);
2010-10-28, by wenzelm
added Exn.interruptible_capture, which reraises interrupts as required by user-code (when Exn.capture is not immediately followed by Exn.release);
2010-10-28, by wenzelm
eliminated dead code;
2010-10-28, by wenzelm
tuned white-space;
2010-10-28, by wenzelm
merged
2010-10-28, by nipkow
added lemmas about listrel(1)
2010-10-28, by nipkow
tuned;
2010-10-28, by wenzelm
merged
2010-10-28, by wenzelm
support non-identifier-like fact names in Sledgehammer (e.g., "my lemma") by quoting them
2010-10-28, by blanchet
merged
2010-10-28, by blanchet
clear identification
2010-10-28, by blanchet
clear identification;
2010-10-28, by blanchet
clear identification
2010-10-28, by blanchet
reintroduced Auto Try, but this time really off by default -- and leave some classical+simp reasoners out for Auto Try (but keep them for Try)
2010-10-27, by blanchet
do not let Metis be confused by higher-order reasoning leading to literals of the form "~ ~ p", which are really the same as "p"
2010-10-27, by blanchet
generalize to handle any prover (not just E)
2010-10-27, by blanchet
merged
2010-10-27, by huffman
make domain package work with non-cpo argument types
2010-10-27, by huffman
make op -->> infixr, to match op --->
2010-10-27, by huffman
use Named_Thms instead of Theory_Data for some domain package theorems
2010-10-26, by huffman
change types of ML commands add_domain, add_new_domain to take 'sort' instead of 'string option'
2010-10-26, by huffman
use Term.add_tfreesT
2010-10-26, by huffman
rename case combinators generated by domain package to 'foo_case' instead of 'foo_when'
2010-10-24, by huffman
rename constant 'one_when' to 'one_case'
2010-10-24, by huffman
merged
2010-10-27, by haftmann
sorting: avoid _key suffix if lemma applies both to simple and generalized variant; generalized insort_insert to insort_insert_key; additional lemmas
2010-10-27, by haftmann
regenerated keyword file
2010-10-27, by krauss
made SML/NJ happy
2010-10-27, by boehmes
adapted SMT solver error handling to reflect latest changes in "SMT_Solver"
2010-10-26, by blanchet
better list of irrelevant SMT constants
2010-10-26, by blanchet
if "debug" is on, print list of relevant facts (poweruser request);
2010-10-26, by blanchet
standardize on "fact" terminology (vs. "axiom" or "theorem") in Sledgehammer -- but keep "Axiom" in the lower-level "ATP_Problem" module
2010-10-26, by blanchet
"Nitpick" -> "Sledgehammer";
2010-10-26, by blanchet
merge
2010-10-26, by blanchet
merged
2010-10-26, by blanchet
remove needless context argument;
2010-10-26, by blanchet
use proper context
2010-10-26, by boehmes
trace assumptions before giving them to the SMT solver
2010-10-26, by boehmes
capture out-of-memory warnings of Z3 and turn them into proper exceptions; be more precise about SMT solver run-time: return NONE instead of ~1
2010-10-26, by boehmes
honor choice of either local or remote SMT solver only for smt_filter and keep default behaviour for the SMT tactic; omit messages when running smt_filter
2010-10-26, by boehmes
include ATP in theory List -- avoid theory edge by-passing the prominent list theory
2010-10-26, by haftmann
fixed typo
2010-10-26, by krauss
merged
2010-10-26, by blanchet
merged
2010-10-26, by blanchet
put theorems added using "add:" at the beginning of the list returned by the relevance filter, so that they don't get truncated away
2010-10-26, by blanchet
tuning
2010-10-26, by blanchet
merged
2010-10-26, by haftmann
consider base sorts of superclasses simultaneously during processing of class specification -- avoids clash of different base sorts
2010-10-26, by haftmann
more general treatment of type argument in code certificates for operations on abstract types
2010-10-26, by haftmann
partial_function is a declaration command
2010-10-26, by haftmann
merged
2010-10-26, by blanchet
proper error handling for SMT solvers in Sledgehammer
2010-10-26, by blanchet
NEWS
2010-10-26, by krauss
merge
2010-10-26, by blanchet
integrated "smt" proof method with Sledgehammer
2010-10-26, by blanchet
fixed confusion introduced in 008dc2d2c395
2010-10-26, by krauss
merged
2010-10-26, by blanchet
reverted e7a80c6752c9 -- there's not much point in putting a diagnosis tool (as opposed to a proof method) in Plain, but more importantly Sledgehammer must be in Main to use SMT solvers
2010-10-26, by blanchet
merged
2010-10-26, by haftmann
tuned
2010-10-26, by haftmann
merged
2010-10-26, by krauss
use partial_function instead of MREC combinator; curried rev'
2010-10-26, by krauss
added Heap monad instance of partial_function package
2010-10-26, by krauss
added Spec_Rule declaration to partial_function
2010-10-26, by krauss
basic documentation for command partial_function
2010-10-26, by krauss
remove outdated "(otherwise)" syntax from manual
2010-10-26, by krauss
declare recursive equation as ".simps", in accordance with other packages
2010-10-26, by krauss
merged
2010-10-26, by haftmann
dropped accidental doubled computation
2010-10-26, by haftmann
optionally force the remote version of an SMT solver to be executed
2010-10-26, by boehmes
tuned
2010-10-26, by boehmes
added a mode to only filter assumptions used in a Z3 proof (in which no proof reconstruction is performed)
2010-10-26, by boehmes
changed SMT configuration options; updated SMT certificates
2010-10-26, by boehmes
joined setup of SMT solvers in one place; turned Z3-specific options into SMT options (renamed configuration options from z3_* to smt_*); more detailed SMT exception; improved SMT filter interface
2010-10-26, by boehmes
keep track of theorems initially given to SMT (even if they are rewritten); provide interface to filter theorems necessary for SMT proofs
2010-10-26, by boehmes
merged
2010-10-26, by blanchet
merge
2010-10-26, by blanchet
clearer error messages
2010-10-26, by blanchet
renaming
2010-10-26, by blanchet
back again to non-Apple font rendering (cf. 4977324373f2);
2010-10-28, by wenzelm
dock isabelle-session at bottom (again, cf. 37bdc2220cf8) to ensure that controls are fully visible;
2010-10-28, by wenzelm
disable broken popups for now;
2010-10-26, by wenzelm
tuned;
2010-10-26, by wenzelm
do not handle arbitrary exceptions;
2010-10-26, by wenzelm
merged
2010-10-26, by wenzelm
Code_Runtime.trace
2010-10-26, by haftmann
proper markup of uninterpreted ML text as @{ML_text}, not @{verbatim};
2010-10-26, by wenzelm
merged
2010-10-26, by wenzelm
improved English
2010-10-26, by blanchet
whitespace tuning
2010-10-26, by blanchet
no need to encode theorem number twice in skolem names
2010-10-26, by blanchet
tuning
2010-10-26, by blanchet
make SML/NJ happy
2010-10-26, by blanchet
relaxing the filtering condition for getting specifications from Spec_Rules
2010-10-25, by bulwahn
adding new predicate compiler files to the IsaMakefile
2010-10-25, by bulwahn
using mode_eq instead of op = for lookup in the predicate compiler
2010-10-25, by bulwahn
renaming split_modeT' to split_modeT
2010-10-25, by bulwahn
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
avoid using Global_Theory.get_thm
2010-10-14, by huffman
include iso_info as part of constr_info type
2010-10-14, by huffman
remove function Domain_Theorems.theorems; bind theorem names directly from Domain_Constructors.add_domain_constructors
2010-10-14, by huffman
add take_strict_thms field to take_info type
2010-10-14, by huffman
add record type synonym 'constr_info'
2010-10-14, by huffman
add function take_theorems
2010-10-14, by huffman
add type annotation to avoid warning
2010-10-14, by huffman
cleaned up Fun_Cpo.thy; deprecated a few theorem names
2010-10-13, by huffman
edit comments
2010-10-13, by huffman
remove unneeded lemmas Lift_exhaust, Lift_cases
2010-10-12, by huffman
move lemmas from Lift.thy to Cfun.thy
2010-10-12, by huffman
cleaned up Adm.thy
2010-10-12, by huffman
remove unneeded lemmas from Fun_Cpo.thy
2010-10-12, by huffman
remove unused lemmas
2010-10-12, by huffman
reformulate lemma cont2cont_lub and move to Cont.thy
2010-10-12, by huffman
remove unused lemmas cont_fst_snd_D1, cont_fst_snd_D2
2010-10-12, by huffman
new theorem names: fun_below_iff, fun_belowI, cfun_eq_iff, cfun_eqI, cfun_below_iff, cfun_belowI
2010-10-11, by huffman
rename Ffun.thy to Fun_Cpo.thy
2010-10-11, by huffman
remove unused constant 'directed'
2010-10-11, by huffman
add HOLCF/Library/Defl_Bifinite.thy, which proves instance defl :: bifinite
2010-10-11, by huffman
merged
2010-10-15, by paulson
prevention of self-referential type environments
2010-10-15, by paulson
FSet: definition changes propagated from Nominal and more use of 'descending' tactic
2010-10-15, by Cezary Kaliszyk
FSet tuned
2010-10-15, by Cezary Kaliszyk
FSet: give names to respectfulness theorems, rename list_all2_refl to avoid clash
2010-10-15, by Cezary Kaliszyk
NEWS
2010-10-14, by krauss
removed output syntax "'a ~=> 'b" for "'a => 'b option"
2010-10-10, by krauss
reactivated
2010-10-13, by krauss
slightly more robust proof
2010-10-12, by krauss
renamed type and constant 'sfp' to 'defl'; replaced syntax SFP('a) with DEFL('a)
2010-10-11, by huffman
merged
2010-10-11, by huffman
move all bifinite class instances to Bifinite.thy
2010-10-09, by huffman
rename class 'sfp' to 'bifinite'
2010-10-08, by huffman
move stuff from Algebraic.thy to Bifinite.thy and elsewhere
2010-10-07, by huffman
add lemma typedef_ideal_completion
2010-10-07, by huffman
remove unused lemmas
2010-10-07, by huffman
remove Infinite_Set from ROOT.ML
2010-10-07, by huffman
remove some junk that made it in by accient
2010-10-07, by huffman
"setup" in theory
2010-10-11, by blanchet
added "trace_meson" configuration option, replacing old-fashioned reference
2010-10-11, by blanchet
added "trace_metis" configuration option, replacing old-fashioned references
2010-10-11, by blanchet
do not mention unqualified names, now that 'global' and 'local' are gone
2010-10-10, by krauss
simplified proof
2010-10-10, by nipkow
avoid generating several formulas with the same name ("tfrees")
2010-10-10, by blanchet
major reorganization/simplification of HOLCF type classes:
2010-10-06, by huffman
add lemma finite_deflation_intro
2010-10-05, by Brian Huffman
add lemmas finite_deflation_imp_compact, cast_below_cast_iff
2010-10-05, by Brian Huffman
move lemmas to Deflation.thy
2010-10-05, by Brian Huffman
simplify proofs of powerdomain inequalities
2010-10-05, by Brian Huffman
new lemmas about lub
2010-10-04, by huffman
define is_ub predicate using bounded quantifier
2010-10-04, by huffman
minimize theory imports
2010-10-02, by huffman
added lemmas to List_Cpo.thy
2010-10-01, by huffman
new_domain emits proper error message when a constructor argument type does not have sort 'rep'
2010-09-30, by huffman
move code from "Metis_Tactics" to "Metis_Reconstruct"
2010-10-06, by blanchet
merged
2010-10-06, by blanchet
qualify "Meson." and "Metis." constants so that the ML files can be reloaded later (e.g. for testing/development)
2010-10-06, by blanchet
get rid of function that duplicates existing Pure functionality
2010-10-06, by blanchet
remove needless fact
2010-10-06, by blanchet
added a few FIXMEs
2010-10-06, by blanchet
tuned comments
2010-10-05, by blanchet
document latest changes to Meson/Metis/Sledgehammer
2010-10-05, by blanchet
remove needless Metis facts
2010-10-05, by blanchet
hide one more name
2010-10-05, by blanchet
qualify names
2010-10-05, by blanchet
hide uninteresting MESON/Metis constants and facts and remove "meson_" prefix to (now hidden) fact names
2010-10-05, by blanchet
clean up debugging output
2010-10-05, by blanchet
factor out "ATP" from "Sledgehammer" (cf. "SAT" vs. "Refute", etc.) -- the theories now reflect the directory structure
2010-10-05, by blanchet
got rid of overkill "meson_choice" attribute;
2010-10-05, by blanchet
more explicit name
2010-10-05, by blanchet
factor out "Meson_Tactic" from "Meson_Clausify"
2010-10-05, by blanchet
tuning
2010-10-04, by blanchet
move Metis into Plain
2010-10-04, by blanchet
added "Meson" theory to Makefile
2010-10-04, by blanchet
update authors
2010-10-04, by blanchet
remove Meson from Hilbert_Choice
2010-10-04, by blanchet
remove Meson from Sledgehammer
2010-10-04, by blanchet
move Meson to Plain
2010-10-04, by blanchet
move MESON files together
2010-10-04, by blanchet
paramify new skolems just like old ones (cf. reveal_old_skolem_terms)
2010-10-04, by blanchet
fixed two bugs in new skolemizer: instantiations now take types into consideration, and rotate_tac is given the proper offset
2010-10-04, by blanchet
correctly handle multiple copies of the same axiom with the same types
2010-10-04, by blanchet
put two operations in the right order
2010-10-04, by blanchet
reintroduce old "unify_prem_with_concl" code to avoid reaching unification bound + primitive handling for polymorphism
2010-10-04, by blanchet
apply "assume_tac" directly on the right assumption, using "rotate_tac" -- this ensures that the desired unifications are performed
2010-10-04, by blanchet
instantiate foralls and release exists in the order described by the topological order
2010-10-04, by blanchet
reverted 0bfaaa81fc62, since "Thm.rename_boundvars" can't be relied upon to give unique names to bound variables
2010-10-04, by blanchet
renamed internal function
2010-10-04, by blanchet
hack in MESON to make it less likely that variables (e.g. "x") get renamed (e.g. "xa") when resolving
2010-10-04, by blanchet
tuned header
2010-10-06, by haftmann
tuned
2010-10-05, by krauss
force less agressively
2010-10-05, by krauss
lexicographic_order: replace parallel map with laziness to avoid wasting cycles on proofs that are not needed
2010-10-05, by krauss
removed complicated (and rarely helpful) error reporting
2010-10-05, by krauss
discontinued continuations to simplify control flow; dropped optimization in scnp
2010-10-05, by krauss
use Cache structure instead of passing tables around explicitly
2010-10-05, by krauss
merged
2010-10-05, by haftmann
lemmas fold_commute and fold_commute_apply
2010-10-05, by haftmann
spelling
2010-05-07, by krauss
adjusted to inductive characterization of sorted
2010-10-04, by haftmann
tuned whitespace
2010-10-04, by haftmann
turned distinct and sorted into inductive predicates: yields nice induction principles for free; more elegant proofs
2010-10-04, by haftmann
turned distinct and sorted into inductive predicates: yields nice induction principles for free
2010-10-04, by haftmann
turned distinct and sorted into inductive predicates: yields nice induction principles for free; more elegant proofs
2010-10-04, by haftmann
some Poly/ML-specific debugging code escaped in the wild -- comment it out
2010-10-02, by blanchet
merged
2010-10-01, by haftmann
avoid antiquotation processing for code_reflect; moved ML_Context.value to Code_Runtime
2010-10-01, by haftmann
moved ML_Context.value to Code_Runtime
2010-10-01, by haftmann
constant `contents` renamed to `the_elem`
2010-10-01, by haftmann
merged
2010-10-01, by blanchet
tune whitespace
2010-10-01, by blanchet
rename bound variables after skolemizing, if the axiom of choice is available
2010-10-01, by blanchet
tuning
2010-10-01, by blanchet
rename quantified variables earlier in the new skolemizer, to ensure consistent naming later (in the absence of the choice axiom)
2010-10-01, by blanchet
tune bound names
2010-10-01, by blanchet
merged
2010-10-01, by blanchet
avoid dependency on "int"
2010-10-01, by blanchet
make "cnf_axiom" work (after a fashion) in the absence of the axiom of choice
2010-10-01, by blanchet
added "meson_choice" attribute as a step towards making (less powerful versions of) Meson/Metis/Sledgehammer work without the axiom of choice
2010-10-01, by blanchet
compute quantifier dependency graph in new skolemizer
2010-10-01, by blanchet
tuning
2010-10-01, by blanchet
compute substitutions in new skolemizer
2010-10-01, by blanchet
encode axiom number and cluster number in all zapped quantifiers to help discharging new skolemizer assumptions
2010-09-30, by blanchet
reintroduced code that keeps track of whether the Isabelle and Metis proofs are in sync -- generalized to work with the new skolemizer
2010-09-30, by blanchet
encode number of skolem assumptions in them, for more efficient retrieval later
2010-09-30, by blanchet
move functions closer to where they're used
2010-09-30, by blanchet
Skolemizer tweaking
2010-09-30, by blanchet
"meson_new_skolemizer" -> "metis_new_skolemizer" option (since Meson doesn't support the new skolemizer (yet))
2010-09-29, by blanchet
finished renaming file and module
2010-09-29, by blanchet
rename file
2010-09-29, by blanchet
ignore Skolem assumption (if any)
2010-09-29, by blanchet
second step in introducing the new Skolemizer -- notably, added procedure for discharging Skolem assumptions
2010-09-29, by blanchet
first step towards a new skolemizer that doesn't require "Eps"
2010-09-29, by blanchet
cumulative update of generated files (since bf164c153d10);
2010-10-22, by wenzelm
removed ML_old.thy, which is largely superseded by ML.thy;
2010-10-22, by wenzelm
more on "Canonical argument order";
2010-10-22, by wenzelm
cover @{Isar.state};
2010-10-22, by wenzelm
more on "Style and orthography";
2010-10-22, by wenzelm
more on "Naming conventions";
2010-10-22, by wenzelm
tuned;
2010-10-22, by wenzelm
more on "Style and orthography";
2010-10-21, by wenzelm
more refs;
2010-10-21, by wenzelm
preliminary material on "Concrete syntax and type-checking";
2010-10-21, by wenzelm
more on "Association lists", based on more succinct version of older material;
2010-10-20, by wenzelm
clarified "lists as a set-like container";
2010-10-20, by wenzelm
more robust treatment of "op IDENT";
2010-10-19, by wenzelm
more on messages;
2010-10-19, by wenzelm
more on synchronized variables;
2010-10-19, by wenzelm
tuned;
2010-10-19, by wenzelm
more robust index_ML antiquotations: guess name from text (affects infixes and type constructors in particular);
2010-10-19, by wenzelm
misc tuning;
2010-10-19, by wenzelm
somewhat modernized version of "Thread-safe programming";
2010-10-18, by wenzelm
more robust examples: explicit @{assert} instead of unchecked output;
2010-10-18, by wenzelm
more on "Configuration options";
2010-10-18, by wenzelm
tuned;
2010-10-18, by wenzelm
more on "Basic data types";
2010-10-18, by wenzelm
more on "Integers";
2010-10-17, by wenzelm
use continental paragraph style, which works better with mixture of (in)formal text;
2010-10-17, by wenzelm
robustified "warn" environment if \parindent is zero (e.g. within itemize, description etc.);
2010-10-17, by wenzelm
more on "Basic ML data types";
2010-10-16, by wenzelm
more robust treatment of symbolic indentifiers (which may contain colons);
2010-10-16, by wenzelm
more examples;
2010-10-16, by wenzelm
tuned;
2010-10-16, by wenzelm
more on "Exceptions";
2010-10-16, by wenzelm
more on "Exceptions";
2010-10-15, by wenzelm
more examples;
2010-10-15, by wenzelm
tuned chapter arrangement;
2010-10-15, by wenzelm
more examples;
2010-10-15, by wenzelm
moved bind_thm(s) to implementation manual;
2010-10-15, by wenzelm
more on "Attributes";
2010-10-14, by wenzelm
misc tuning and clarification;
2010-10-14, by wenzelm
more on "Proof methods";
2010-10-13, by wenzelm
examples in Isabelle/HOL;
2010-10-13, by wenzelm
more on Proof.theorem;
2010-10-13, by wenzelm
tuned;
2010-10-13, by wenzelm
more examples;
2010-10-12, by wenzelm
more on "Isar language elements";
2010-10-12, by wenzelm
more examples;
2010-10-11, by wenzelm
more refs;
2010-10-11, by wenzelm
misc tuning;
2010-10-11, by wenzelm
removed some obsolete reference material;
2010-10-10, by wenzelm
cover some more theory operations;
2010-10-10, by wenzelm
note on Isabelle file specifications;
2010-10-10, by wenzelm
modernized version of "Message output channels";
2010-10-10, by wenzelm
removed some really old reference material;
2010-10-10, by wenzelm
more examples;
2010-10-09, by wenzelm
various concrete ML antiquotations;
2010-10-09, by wenzelm
prefer checked antiquotations;
2010-10-09, by wenzelm
clarified tag markup;
2010-10-09, by wenzelm
more on ML antiquotations;
2010-10-08, by wenzelm
keep normal size for %mlref tag;
2010-10-08, by wenzelm
basic setup for ML antiquotations -- with rail diagrams;
2010-10-08, by wenzelm
eliminated "Toplevel control", which belongs to TTY/ProofGeneral model;
2010-10-08, by wenzelm
eliminated fancy \ML logo for the sake of simpler source text (less dependence on LaTeX);
2010-10-08, by wenzelm
misc tuning;
2010-10-08, by wenzelm
more on Isabelle/ML;
2010-10-07, by wenzelm
basic setup for Chapter 0: Isabelle/ML;
2010-10-07, by wenzelm
minor tuning and updating;
2010-10-07, by wenzelm
made SML/NJ happy;
2010-10-01, by wenzelm
merged
2010-10-01, by wenzelm
use module integer for Eval
2010-10-01, by haftmann
check whole target hierarchy for existing reserved symbols
2010-10-01, by haftmann
added polyml_as_definition -- using external SML files as substitute for proper definitions -- only for polyml!
2010-10-01, by haftmann
tuned default "Prover Session" perspective;
2010-10-01, by wenzelm
eliminated ancient OldTerm.term_frees;
2010-10-01, by wenzelm
more antiquotations;
2010-10-01, by wenzelm
simplified outer syntax setup;
2010-10-01, by wenzelm
chop_while replace drop_while and take_while
2010-10-01, by haftmann
merged
2010-10-01, by haftmann
take_while, drop_while
2010-09-30, by haftmann
rename cont2cont_split to cont2cont_prod_case; add lemmas prod_contI, prod_cont_iff; simplify some proofs
2010-09-30, by huffman
fixrec: rename match_cpair to match_Pair
2010-09-30, by huffman
remove code for obsolete 'fixpat' command
2010-09-15, by huffman
clean up definition of compile_pat function
2010-09-15, by huffman
rename some fixrec pattern-match compilation functions
2010-09-15, by huffman
adding example for case expressions
2010-09-30, by bulwahn
applying case beta reduction to case term before matching in predicate compile function flattening; moving case beta reduction function to Predicate_Compile_Aux
2010-09-30, by bulwahn
merged
2010-09-30, by bulwahn
adapting manual configuration in examples
2010-09-30, by bulwahn
finding the counterexample with different options (manually limited precisely, manually limited global, automatically limited global)
2010-09-30, by bulwahn
adding option to globally limit the prolog execution
2010-09-30, by bulwahn
removing dead code
2010-09-30, by bulwahn
value uses bare compiler invocation: generated code does not contain antiquotations
2010-09-30, by haftmann
updated files to recent changes
2010-09-30, by haftmann
corrected subsumption check: arguments have been reversed; addition of default equations to non-default equations is identity
2010-09-30, by haftmann
tuned
2010-09-30, by haftmann
merged
2010-09-30, by haftmann
redundancy check: drop trailing Var arguments (avoids eta problems with equations)
2010-09-29, by haftmann
merged
2010-09-29, by wenzelm
removing obsolete distinction between prod_case and other case expressions after merging of split and prod_case (d3daea901123) in predicate compiler
2010-09-29, by bulwahn
merged
2010-09-29, by bulwahn
adding splitting of conjuncts in assumptions as forward rule on theorems; replacing term transformation for splitting conjuncts by theorem transformation; removing obsolete functions; tuned
2010-09-29, by bulwahn
added test case for predicate arguments in higher-order argument position
2010-09-29, by bulwahn
improving the compilation to handle predicate arguments in higher-order argument positions
2010-09-29, by bulwahn
added a test case to Predicate_Compile_Tests
2010-09-29, by bulwahn
putting the last step of the proof in a TRY block to handle the case that the simplifier already solved the goal
2010-09-29, by bulwahn
backed out my old attempt at single_hyp_subst_tac (67cd6ed76446)
2010-09-29, by krauss
scala is reserved identifier
2010-09-29, by haftmann
platform-sensitive contrib paths for ghc, ocaml
2010-09-29, by haftmann
fact listsum now names listsum_foldl
2010-09-29, by haftmann
delete code lemma explicitly
2010-09-29, by haftmann
moved old_primrec source to nominal package, where it is still used
2010-09-29, by haftmann
dropped old primrec package
2010-09-28, by haftmann
merged
2010-09-28, by haftmann
localized listsum
2010-09-28, by haftmann
lemma listsum_conv_fold
2010-09-28, by haftmann
merged
2010-09-28, by haftmann
NEWS
2010-09-28, by haftmann
dropped syntax for old primrec package
2010-09-28, by haftmann
modernized session
2010-09-28, by haftmann
merged
2010-09-28, by bulwahn
using SUBPROOF to ensure that rewriting is not done on the further subgoals of proof
2010-09-28, by bulwahn
avoiding instable rotate_tac and using the nice Subgoal.FOCUS_PREMS instead
2010-09-28, by bulwahn
adding test case for interpretation of arguments that are predicates simply as input
2010-09-28, by bulwahn
only modes but not types are used to destruct terms and types; this allows to interpret arguments that are predicates simply as input
2010-09-28, by bulwahn
weakening check for higher-order relations, but adding check for consistent modes
2010-09-28, by bulwahn
handling higher-order relations in output terms; improving proof procedure; added test case
2010-09-28, by bulwahn
renaming use_random to use_generators in the predicate compiler
2010-09-28, by bulwahn
fixed a typo that caused the preference of non-random modes to be ignored
2010-09-28, by bulwahn
merged
2010-09-28, by haftmann
modernized primrecs
2010-09-28, by haftmann
modernized session
2010-09-28, by haftmann
consolidated tupled_lambda; moved to structure HOLogic
2010-09-28, by krauss
added dependency to base image to ensure that the doc test actually rebuilds the tutorial
2010-09-28, by haftmann
no longer declare .psimps rules as [simp].
2010-09-28, by krauss
added dependency to base images to ensure that the doc test actually rebuilds the tutorials
2010-09-28, by krauss
removed unnecessary reference poking (cf. f45d332a90e3)
2010-09-28, by krauss
merged
2010-09-28, by haftmann
consider quick_and_dirty option before loading theory
2010-09-28, by haftmann
dropped obsolete mk_tcl
2010-09-28, by krauss
make SML/NJ happy
2010-09-28, by blanchet
merged
2010-09-27, by haftmann
combine quote and typewriter tag; typewriter considers isa@parindent
2010-09-27, by haftmann
combine quote and typewriter/tt tag
2010-09-27, by haftmann
combine quote and typewriter tag; typewriter considers isa@parindent
2010-09-27, by haftmann
combine quote and typewriter tag
2010-09-27, by haftmann
CONTROL-mouse management: handle windowDeactivated as well;
2010-09-29, by wenzelm
CONTROL-mouse management: handle windowIconified;
2010-09-28, by wenzelm
basic support for message popups via HTML_Panel;
2010-09-28, by wenzelm
tuned default perspective;
2010-09-28, by wenzelm
tuned README;
2010-09-28, by wenzelm
more defensive overview.paintComponent: avoid potential crash due to buffer change while painting;
2010-09-28, by wenzelm
tuned README;
2010-09-28, by wenzelm
more uniform init/exit model/view in session_manager, trading race wrt. session.phase for race wrt. global editor state;
2010-09-28, by wenzelm
moved "auto-start" to options panel;
2010-09-27, by wenzelm
renamed raw output primitives to emphasize their meaning -- not to be used in user-space;
2010-09-27, by wenzelm
added Standard_System.unzip (for platform file-system);
2010-09-27, by wenzelm
bulk read: observe EOF protocol more carefully -- 0 counts as successful read;
2010-09-27, by wenzelm
tuned whitespace;
2010-09-27, by wenzelm
merged
2010-09-27, by wenzelm
lemma remdups_map_remdups
2010-09-27, by haftmann
lemma remdups_list_of_dlist
2010-09-27, by haftmann
merged
2010-09-27, by bulwahn
adopting example
2010-09-27, by bulwahn
adding further tracing messages; tuned
2010-09-27, by bulwahn
handling nested cases more elegant by requiring less new constants
2010-09-27, by bulwahn
merged
2010-09-27, by blanchet
renamed function
2010-09-27, by blanchet
rename "Clausifier" to "Meson_Clausifier" and merge with "Meson_Tactic"
2010-09-27, by blanchet
comment out Auto Try until issues are resolved (automatically on by default even though the code says off; thread that continues in the background)
2010-09-27, by blanchet
remove needless flag
2010-09-27, by blanchet
added hint on reference equality
2010-09-27, by haftmann
treat equality on refs and arrays as primitive operation
2010-09-27, by haftmann
corrected OCaml operator precedence
2010-09-27, by haftmann
corrected scope of closure
2010-09-27, by haftmann
merged
2010-09-27, by haftmann
separate quote tag from tt tag
2010-09-27, by haftmann
separate quote tag from tt tag
2010-09-24, by haftmann
make SML/NJ happy
2010-09-25, by blanchet
some more options to robustify posix_untar;
2010-09-27, by wenzelm
more efficient posix_untar -- avoid really slow java.util.zip.GZIPInputStream;
2010-09-27, by wenzelm
back to UseQuartz=true -- used to be default on Apple Java 1.5;
2010-09-27, by wenzelm
raw_untar.raw_execute with native cwd, to avoid cross-platform complications;
2010-09-26, by wenzelm
added Standard_System.raw_untar;
2010-09-26, by wenzelm
some markup for inner syntax tokens;
2010-09-26, by wenzelm
tuned signatures and messages;
2010-09-26, by wenzelm
Session_Dockable: more startup controls;
2010-09-25, by wenzelm
simplified / clarified Session.Phase;
2010-09-25, by wenzelm
more precise treatment of backgrounds vs. rectangles;
2010-09-25, by wenzelm
tuned mk_fifo;
2010-09-25, by wenzelm
tuned signature;
2010-09-25, by wenzelm
tuned border;
2010-09-24, by wenzelm
more informative Session.Phase;
2010-09-24, by wenzelm
merged
2010-09-24, by wenzelm
merged
2010-09-24, by haftmann
tuned schema table
2010-09-24, by haftmann
tuned warning_color;
2010-09-24, by wenzelm
tuned error_color;
2010-09-24, by wenzelm
some attempts to improve visual appearance of bad text;
2010-09-24, by wenzelm
clarified @{type} antiquotation: abbreviations and nonterminals count as "syntactic", disallow TFrees;
2010-09-24, by wenzelm
updated generated file;
2010-09-24, by wenzelm
modernized structure Ord_List;
2010-09-24, by wenzelm
isatest: indicate Isabelle version;
2010-09-24, by wenzelm
actually handle Type.TYPE_MATCH, not arbitrary exceptions;
2010-09-24, by wenzelm
merged
2010-09-24, by wenzelm
prefer typewrite tag over raw latex environment
2010-09-24, by haftmann
avoid fragile tranclp syntax; corrected resolution; corrected typo
2010-09-24, by haftmann
merged
2010-09-24, by wenzelm
use typewriter tag instead of bare environment
2010-09-24, by haftmann
dropped dead code
2010-09-24, by haftmann
always add trailing newline for presentation
2010-09-24, by haftmann
corrected omission
2010-09-24, by haftmann
fixed small font size fore typewriter text
2010-09-24, by haftmann
merged
2010-09-24, by haftmann
load theory explicitly
2010-09-24, by haftmann
merge
2010-09-24, by blanchet
make SML/NJ happier -- temporary solution until Metis is fixed upstream
2010-09-24, by blanchet
merged
2010-09-24, by bulwahn
being a little less strict than in 2e06dad03dd3
2010-09-24, by bulwahn
quotient package: respectfulness and preservation of identity.
2010-09-24, by Cezary Kaliszyk
merged
2010-09-23, by haftmann
merged
2010-09-23, by haftmann
removed superfluous output_typewriter from cs 65064e8f269
2010-09-23, by haftmann
more idiomatic handling of latex typewriter type setting
2010-09-23, by haftmann
more canonical type setting of type writer code examples
2010-09-23, by haftmann
resynchronize isabelle.sty
2010-09-23, by haftmann
reverted cs 5aced2f43837 -- no need for hardwired latex command here
2010-09-23, by haftmann
reverted cs 07549694e2f1 -- use re-printing with current print mode instead after code assembly, avoid Latex.output_typewriter
2010-09-23, by haftmann
reverted cs 07549694e2f1
2010-09-23, by haftmann
shifted abstraction over imperative print mode
2010-09-23, by haftmann
removing unneccessary expansion procedure for elimination rules; removing obsolete elim preprocessing; tuned
2010-09-23, by bulwahn
moving the preprocessing of introduction rules after the code_pred command; added tuple expansion preprocessing of elimination rule
2010-09-23, by bulwahn
exporting the generic version instead of the context version in quickcheck
2010-09-23, by bulwahn
splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
2010-09-23, by bulwahn
adding a mutual recursive example for named alternative rules for the predicate compiler
2010-09-23, by bulwahn
handling TYPE_MATCH error by raising user error message if user gives introduction rules with mismatching types
2010-09-23, by bulwahn
improving naming of assumptions in code_pred
2010-09-23, by bulwahn
adding check if user-given modes match type of predicates; removed useless function expand_tuples_elim
2010-09-23, by bulwahn
handling equivalences smarter in the predicate compiler
2010-09-23, by bulwahn
removing duplicate rewrite rule from simpset in predicate compiler
2010-09-23, by bulwahn
rewriting function mk_Eval_of in predicate compiler
2010-09-23, by bulwahn
merged
2010-09-23, by haftmann
improved and tuned external codegen tool
2010-09-23, by haftmann
make SML/NJ happy
2010-09-23, by blanchet
CONTRIBUTORS and NEWS
2010-09-23, by haftmann
corrections and tuning
2010-09-23, by haftmann
merged
2010-09-22, by haftmann
merged
2010-09-22, by haftmann
merged
2010-09-22, by haftmann
tuned
2010-09-22, by haftmann
persistent session-panel.selection;
2010-09-24, by wenzelm
slightly more robust EditBus plumbing wrt. Document_View/Document_Model;
2010-09-24, by wenzelm
permissive exit;
2010-09-24, by wenzelm
added Session_Dockable.session_phase label;
2010-09-24, by wenzelm
separate Plugin.init_model;
2010-09-23, by wenzelm
simplified Session.Phase;
2010-09-23, by wenzelm
tuned messages -- cf. Admin/MacOS/App1;
2010-09-23, by wenzelm
tuned dialog;
2010-09-23, by wenzelm
explicit Session.Phase indication with associated event bus;
2010-09-23, by wenzelm
tuned signature;
2010-09-23, by wenzelm
Plugin.stop: refrain from invalidating Isabelle.session -- some actors/dockables out there might still refer to it;
2010-09-23, by wenzelm
tuned;
2010-09-23, by wenzelm
manage persistent syslog via Session, not Isabelle_Process;
2010-09-23, by wenzelm
tuned prover message categorization;
2010-09-23, by wenzelm
tuned Isabelle_Sidekick.complete: lock buffer, depend on document model;
2010-09-23, by wenzelm
tuned message;
2010-09-23, by wenzelm
Command.accumulate: refrain from adding tracing messages to markup tree -- potential scalability problem;
2010-09-22, by wenzelm
Snapshot.convert/revert: explicit error report to isolate sporadic crash;
2010-09-22, by wenzelm
make compiler doubly sure;
2010-09-22, by wenzelm
isabelle-process: less verbose no-commit mode;
2010-09-22, by wenzelm
tuned message;
2010-09-22, by wenzelm
tuned panel names and actions;
2010-09-22, by wenzelm
renamed setmp_noncritical to Unsynchronized.setmp to emphasize its meaning;
2010-09-22, by wenzelm
reactivated polyml-5.4.0 -- SVN 1214 fixes a problem with arbitrary precision arithmetic that was triggered by method "approximation" in HOL/Decision_Procs/Approximation_Ex.thy;
2010-09-22, by wenzelm
merged
2010-09-22, by nipkow
more lists lemmas
2010-09-22, by nipkow
merged
2010-09-22, by wenzelm
merged
2010-09-22, by haftmann
tuned text
2010-09-22, by haftmann
sections on @{code} and code_reflect
2010-09-22, by haftmann
formal syntax diagram for code_reflect
2010-09-22, by haftmann
distinguish SML and Eval explicitly
2010-09-22, by haftmann
no_frees_* is subsumed by new framework mechanisms in Code_Preproc
2010-09-21, by haftmann
reject term variables explicitly
2010-09-21, by haftmann
avoid frees and vars in terms to be evaluated by abstracting and applying
2010-09-21, by haftmann
tuned whitespace
2010-09-21, by haftmann
make SML/NJ happier
2010-09-22, by blanchet
more conventional conversion signature
2010-09-21, by haftmann
added nbe paper
2010-09-21, by haftmann
continued section abut evaluation
2010-09-21, by haftmann
make SML/NJ happier
2010-09-21, by blanchet
new lemma
2010-09-21, by nipkow
merged
2010-09-20, by nipkow
new lemmas
2010-09-20, by nipkow
revert b96941dddd04 and c13b4589fddf, which dramatically inflate proof terms
2010-09-20, by blanchet
basic setup for Session_Dockable controls;
2010-09-22, by wenzelm
tuned signature;
2010-09-22, by wenzelm
more content for Session_Dockable;
2010-09-22, by wenzelm
basic support for full document rendering;
2010-09-22, by wenzelm
Session_Dockable: basic syslog output;
2010-09-22, by wenzelm
just one Session.raw_messages event bus;
2010-09-22, by wenzelm
more reactive handling of Isabelle_Process startup errors;
2010-09-22, by wenzelm
eliminated Simple_Thread shorthands that can overlap with full version;
2010-09-22, by wenzelm
main Isabelle_Process via Isabelle_System.Managed_Process;
2010-09-22, by wenzelm
more robust Managed_Process.kill: check after sending signal;
2010-09-22, by wenzelm
more robust lib/scripts/process, with explicit script/no_script mode;
2010-09-22, by wenzelm
Standard_System.with_tmp_file: deleteOnExit to make double sure;
2010-09-22, by wenzelm
refined Isabelle_System.bash_output: pass pid via stdout, separate stdout/stderr;
2010-09-21, by wenzelm
tuned whitespace;
2010-09-21, by wenzelm
tuned;
2010-09-21, by wenzelm
added Standard_System.slurp convenience;
2010-09-21, by wenzelm
added Simple_Thread.future convenience;
2010-09-21, by wenzelm
refined ML/Scala bash wrapper, based on more general lib/scripts/process;
2010-09-20, by wenzelm
tuned;
2010-09-20, by wenzelm
more robust Isabelle_System.rm_fifo: avoid external bash invocation, which might not work in JVM shutdown phase (due to Runtime.addShutdownHook);
2010-09-20, by wenzelm
tuned;
2010-09-20, by wenzelm
added Isabelle_Process.syslog;
2010-09-20, by wenzelm
updated keywords;
2010-09-20, by wenzelm
merged
2010-09-20, by wenzelm
merged
2010-09-20, by haftmann
corrected long-overlooked slip: the Pure equality of a code equation is no part of the code equation itself
2010-09-20, by haftmann
dynamic_eval_conv static_eval_conv: certification of previously unreliably reconstructed evaluated term
2010-09-20, by haftmann
Pure equality is a regular cpde operation
2010-09-20, by haftmann
full palette of dynamic/static value(_strict/exn)
2010-09-20, by haftmann
Factored out ML into separate file
2010-09-20, by haftmann
merged
2010-09-20, by wenzelm
merged
2010-09-20, by blanchet
remove needless exception
2010-09-20, by blanchet
preprocess "Ex" before doing clausification in Metis;
2010-09-20, by blanchet
expand_fun_eq -> fun_eq_iff
2010-09-20, by haftmann
use buffers instead of string concatenation
2010-09-20, by haftmann
renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
2010-09-20, by wenzelm
more antiquotations;
2010-09-20, by wenzelm
added XML.content_of convenience -- cover XML.body, which is the general situation;
2010-09-20, by wenzelm
merged
2010-09-20, by wenzelm
merged
2010-09-20, by haftmann
more accurate exception handling
2010-09-20, by haftmann
merged
2010-09-20, by blanchet
merge tracing of two related modules
2010-09-20, by blanchet
merged
2010-09-20, by blanchet
preprocess "All" before doing clausification in Metis;
2010-09-18, by blanchet
reorder proof methods and take out "best";
2010-09-17, by blanchet
renaming variable name to decrease likelyhood of nameclash
2010-09-20, by bulwahn
code_pred_intro can be used to name facts for the code_pred command
2010-09-20, by bulwahn
replacing temporary hack by checking for environment settings of the component
2010-09-20, by bulwahn
removing unnessary options for code_pred
2010-09-20, by bulwahn
moving renaming_vars to post_processing; removing clone in values and quickcheck of code_prolog
2010-09-20, by bulwahn
removing clone in code_prolog and predicate_compile_quickcheck
2010-09-20, by bulwahn
adjusted
2010-09-20, by haftmann
updated file duplicate
2010-09-20, by haftmann
\\isatypewrite now part of isabelle latex style
2010-09-20, by haftmann
made smlnj happy
2010-09-20, by haftmann
properly parse Z3 error models, including datatypes, and represent function valuations as lambda terms; also normalize Z3 error models
2010-09-19, by boehmes
do not treat natural numbers as a datatype (natural numbers are considered an abstract type with a coercion to integers)
2010-09-19, by boehmes
generalized lemma insort_remove1 to insort_key_remove1
2010-09-17, by haftmann
generalized lemmas multiset_of_insort, multiset_of_sort, properties_for_sort for *_key variants
2010-09-17, by haftmann
merged
2010-09-17, by haftmann
less intermediate data structures
2010-09-17, by haftmann
Isabelle_Process: more robust rendezvous, even without proper blocking on open (Cygwin);
2010-09-20, by wenzelm
simplified Isabelle_System.mk_fifo: inlined script, append PPID and PID uniformly;
2010-09-19, by wenzelm
refined Isabelle_Process startup: emit \002 before rendezvous on fifos, more robust treatment of startup failure with timeout, do not quit() after main loop;
2010-09-19, by wenzelm
back to default fold painter -- Circle looks slightly odd in conjunction with bracket matching;
2010-09-19, by wenzelm
message_actor: more robust treatment of EOF;
2010-09-19, by wenzelm
simplified Isabelle_Process message kinds;
2010-09-19, by wenzelm
recovered basic session stop/restart;
2010-09-18, by wenzelm
simplified fifo handling -- rm_fifo always succeeds without ever blocking;
2010-09-18, by wenzelm
raw_execute: let IOException pass-through unhindered (again);
2010-09-18, by wenzelm
mkfifo: some workaround to ensure reasonably unique id, even on Cygwin where $PPID might fall back on odd default;
2010-09-18, by wenzelm
Isabelle_System.mk_fifo: more robust enumeration of unique names, based on persisting JVM pid (parent of shell process);
2010-09-18, by wenzelm
slightly more robust Isabelle_Process startup -- NB: openening fifo streams synchronizes with other end, which may fail to reach that point;
2010-09-18, by wenzelm
tuned;
2010-09-18, by wenzelm
separate Isabelle.logic_selector;
2010-09-18, by wenzelm
non-editable text area;
2010-09-18, by wenzelm
basic setup for prover session panel;
2010-09-18, by wenzelm
ML_Syntax.print_char: more readable output of some well-known ASCII controls -- this is relevant for ML toplevel pp;
2010-09-17, by wenzelm
discontinued Output.debug, which belongs to early PGIP experiments (b6788dbd2ef9) and causes just too many problems (like spamming the message channel if it is used by more than one module);
2010-09-17, by wenzelm
Isabelle_Markup.overview_color: indicate error / warning messages;
2010-09-17, by wenzelm
some specific message classification;
2010-09-17, by wenzelm
Syntax.read_asts error: report token ranges within message -- no side-effect here;
2010-09-17, by wenzelm
Isabelle_Process: status/report do not require serial numbers;
2010-09-17, by wenzelm
simplified some internal flags using Config.T instead of full-blown Proof_Data;
2010-09-17, by wenzelm
tuned signature of (Context_)Position.report variants;
2010-09-17, by wenzelm
merged
2010-09-17, by wenzelm
merged
2010-09-17, by blanchet
update README
2010-09-17, by blanchet
regenerate "metis.ML"
2010-09-17, by blanchet
fix license
2010-09-17, by blanchet
updated source files with Metis 2.3 (timestamp: 16 Sept. 2010)
2010-09-17, by blanchet
move functions around
2010-09-17, by blanchet
simplify Skolem handling;
2010-09-17, by blanchet
make "subst_translation" more robust w.r.t. type instantiations like {_1234 |-> 'a}
2010-09-17, by blanchet
complete refactoring of Metis along the lines of Sledgehammer
2010-09-16, by blanchet
got caught once again by SML's pattern maching (ctor vs. var)
2010-09-16, by blanchet
added new "Metis_Reconstruct" module, temporarily empty
2010-09-16, by blanchet
rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
2010-09-16, by blanchet
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
2010-09-16, by blanchet
skip some "important" messages
2010-09-16, by blanchet
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
2010-09-16, by blanchet
merged
2010-09-17, by nipkow
added lemmas
2010-09-17, by nipkow
merged
2010-09-17, by haftmann
proper closures for static evaluation; no need for FIXMEs any longer
2010-09-17, by haftmann
refined static_eval_conv_simple; tuned comments
2010-09-17, by haftmann
closures preserve static serializer context for static evaluation; tuned
2010-09-17, by haftmann
closures separate serializer initialization from serializer invocation as far as appropriate
2010-09-17, by haftmann
add full support for datatypes to the SMT interface (only used by Z3 in oracle mode so far); added store to keep track of datatype selector functions
2010-09-17, by boehmes
made sml/nj happy
2010-09-17, by haftmann
merged
2010-09-16, by haftmann
added code_stmts antiquotation from doc-src/more_antiquote.ML
2010-09-16, by haftmann
added output_typewriter from doc-src/more_antiquote.ML
2010-09-16, by haftmann
moved material intro distribution proper
2010-09-16, by haftmann
merged
2010-09-16, by haftmann
merged
2010-09-16, by haftmann
separation of static and dynamic thy context
2010-09-16, by haftmann
adjusted setup
2010-09-16, by haftmann
dynamic and static value computation; built-in evaluation of propositions
2010-09-16, by haftmann
Exn.map_result
2010-09-16, by haftmann
adjusted to changes in Code_Runtime
2010-09-16, by haftmann
merged
2010-09-16, by bulwahn
merged
2010-09-16, by bulwahn
improving replacing higher order arguments to work with tuples
2010-09-16, by bulwahn
adding another context free grammar example for the predicate compiler
2010-09-16, by bulwahn
adding values to show and ensure that values works with complex terms and restores numerals on natural numbers
2010-09-16, by bulwahn
adding restoring of numerals for natural numbers for values command
2010-09-16, by bulwahn
values command for prolog supports complex terms and not just variables
2010-09-16, by bulwahn
adapting examples
2010-09-16, by bulwahn
registering code_prolog as component; using environment variable; adding settings file for prolog code generation
2010-09-16, by bulwahn
adding mode inference to prolog compilation; separate between (ad-hoc) code modifications and system_configuration; adapting quickcheck
2010-09-16, by bulwahn
merged
2010-09-16, by paulson
tidied a few proofs
2010-09-16, by paulson
merged
2010-09-16, by blanchet
avoid code duplication
2010-09-16, by blanchet
tuning
2010-09-16, by blanchet
merge constructors
2010-09-16, by blanchet
factor out the inverse of "nice_atp_problem"
2010-09-16, by blanchet
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
2010-09-16, by blanchet
factored out TSTP/SPASS/Vampire proof parsing;
2010-09-16, by blanchet
prevent exception when calling "Mirabelle.can_apply" on empty proof sequence;
2010-09-16, by blanchet
supply the Metis parameter defaults as argument, instead of patching the Metis sources;
2010-09-16, by blanchet
regenerated "metis.ML"
2010-09-16, by blanchet
streamlined "make_metis"
2010-09-16, by blanchet
put Isabelle-specifics in a "PortableIsabelle" file maintained by us;
2010-09-16, by blanchet
handy little script
2010-09-16, by blanchet
reintroduce missing "critical"s by hand
2010-09-16, by blanchet
MIT license -> BSD License
2010-09-16, by blanchet
copied the unmodified official Metis 2.3 (15 Sept. 2010) sources into Isabelle
2010-09-16, by blanchet
tuned;
2010-09-17, by wenzelm
allow embedded reports in regular prover messages, to avoid side-effects for errors for example;
2010-09-17, by wenzelm
simplified/clarified (Context_)Position.markup/reported_text;
2010-09-17, by wenzelm
eliminated markup "location" in favour of more explicit "no_report", which is actually deleted from messages;
2010-09-17, by wenzelm
Isar "default" step needs to fail for solved problems, for clear distinction of '.' and '..' for example -- amending lapse introduced in 9de4d64eee3b (April 2004);
2010-09-16, by wenzelm
updated generated file;
2010-09-16, by wenzelm
tuned whitespace
2010-09-16, by haftmann
reverse order of datatype declarations so that declarations only depend on already declared datatypes
2010-09-16, by boehmes
merged
2010-09-15, by blanchet
make "metis.ML" building process slightly more robust by eliminating the need for "FILES";
2010-09-15, by blanchet
dropped obsolete src/Tools/random_word.ML -- superseded by src/Tools/Metis/src/Random.sml stemming from the Metis distribution;
2010-09-15, by wenzelm
merged
2010-09-15, by blanchet
document Metis updating procedure
2010-09-15, by blanchet
move "CRITICAL" to "PortableXxx", where it belongs and used to be;
2010-09-15, by blanchet
regenerated "metis.ML"
2010-09-15, by blanchet
update comment
2010-09-15, by blanchet
make "Unprotected concurrency introduces some true randomness." be true;
2010-09-15, by blanchet
fix parsing of higher-order formulas;
2010-09-15, by blanchet
merged
2010-09-15, by haftmann
load code_runtime immediately again
2010-09-15, by haftmann
proper interface for code_reflect
2010-09-15, by haftmann
introduced "holds" as synthetic datatype constructor for "prop"; moved Pure code generator setup to Code_Generator.thy
2010-09-15, by haftmann
merged
2010-09-15, by blanchet
"Metis." -> "Metis_" to reflect change in "metis.ML"
2010-09-15, by blanchet
no need for "metis_env.ML" anymore;
2010-09-15, by blanchet
regenerate "metis.ML", this time without manual hacks
2010-09-15, by blanchet
remove needless file for us
2010-09-15, by blanchet
got rid of three crude regexps from "make_metis"
2010-09-15, by blanchet
more Isabelle-specific changes
2010-09-15, by blanchet
tuning
2010-09-15, by blanchet
rename
2010-09-15, by blanchet
use "Metis_" prefix rather than "Metis" structure;
2010-09-15, by blanchet
no need for TPTP
2010-09-15, by blanchet
put "foldl" and "foldr" in "Useful";
2010-09-15, by blanchet
reintroduce the CRITICAL sections from change 3880d21d6013
2010-09-15, by blanchet
apply Larry's hacks directly to the "src" files;
2010-09-15, by blanchet
"FILES" is not (anymore?) part of the official Metis sources, so move it up
2010-09-15, by blanchet
merged
2010-09-15, by wenzelm
Code_Runtime.value, corresponding to ML_Context.value; tuned
2010-09-15, by haftmann
Code_Runtime.value, corresponding to ML_Context.value
2010-09-15, by haftmann
more accurate dependencies
2010-09-15, by haftmann
code_eval renamed to code_runtime
2010-09-15, by haftmann
merged
2010-09-15, by wenzelm
static nbe conversion
2010-09-15, by haftmann
ignore code cache optionally; corrected scope of term value in static_eval_conv
2010-09-15, by haftmann
ignore code cache optionally
2010-09-15, by haftmann
dropped redundant normal_form command
2010-09-15, by haftmann
more explicit theory name
2010-09-15, by haftmann
more accurate dependencies
2010-09-15, by haftmann
merged
2010-09-15, by haftmann
more clear separation of static compilation and dynamic evaluation
2010-09-15, by haftmann
Document.async_state: some attempts to make this more robust wrt. cancelation of the main transaction -- avoid confusing feedback about pending forks;
2010-09-15, by wenzelm
isatest: reactivated kodkodi and thus HOL-Nitpick_Examples -- being now on a local file system greatly increases the chance that it works;
2010-09-15, by wenzelm
merged
2010-09-15, by haftmann
replaced ML_Context.evaluate by ML_Context.value -- using context data instead of bare metal references
2010-09-15, by haftmann
replaced ML_Context.evaluate by ML_Context.value -- using context data instead of bare metal references; tuned structures
2010-09-15, by haftmann
merge
2010-09-15, by blanchet
compile on SML/NJ
2010-09-15, by blanchet
in debug mode, don't touch "$true" and "$false"
2010-09-15, by blanchet
adding option show_invalid_clauses for a more detailed message when modes are not inferred
2010-09-15, by bulwahn
proposed modes for code_pred now supports modes for mutual predicates
2010-09-15, by bulwahn
merged
2010-09-15, by haftmann
established emerging canonical names *_eqI and *_eq_iff
2010-09-13, by haftmann
moved lemmas map_of_eqI and map_of_eq_dom to Map.thy
2010-09-13, by haftmann
more precise name for activation of improveable syntax
2010-09-13, by haftmann
tuning
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
prefer version 0.6 of Vampire, now that we can parse its output
2010-09-14, by blanchet
fix splitting of proof lines for one-line metis calls;
2010-09-14, by blanchet
finish support for E 1.2 proof reconstruction;
2010-09-14, by blanchet
first step in generalizing to nonnumeric proof step names (e.g. remote Vampire 0.6)
2010-09-14, by blanchet
clarify message
2010-09-14, by blanchet
use same hack as in "Async_Manager" to work around Proof General bug
2010-09-14, by blanchet
export function
2010-09-14, by blanchet
generalize proof reconstruction code;
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
handle relevance filter corner cases more gracefully;
2010-09-14, by blanchet
remove more clutter related to old "fast_descrs" optimization
2010-09-14, by blanchet
Sledgehammer should be called in "prove" mode;
2010-09-14, by blanchet
added a timeout around "try" call in Mirabelle
2010-09-14, by blanchet
adapt examples to latest Nitpick changes + speed them up a little bit
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
eliminate more clutter related to "fast_descrs" optimization
2010-09-14, by blanchet
remove "fast_descs" option from Nitpick;
2010-09-14, by blanchet
fixed bug in the "fast_descrs" optimization;
2010-09-14, by blanchet
speed up helper function
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
rename internal Sledgehammer constant
2010-09-14, by blanchet
merged
2010-09-14, by blanchet
merged
2010-09-13, by blanchet
adapt to latest Metis version
2010-09-13, by blanchet
regenerated "metis.ML" and reintroduced Larry's old hacks manually;
2010-09-13, by blanchet
update scripts
2010-09-13, by blanchet
change license, with Joe Hurd's permission
2010-09-13, by blanchet
new version of the Metis files
2010-09-13, by blanchet
remove old sources
2010-09-13, by blanchet
remove "atoms" from the list of options with default values
2010-09-13, by blanchet
remove unreferenced identifiers
2010-09-13, by blanchet
make Auto Nitpick go through fewer scopes
2010-09-13, by blanchet
move equation up where it's not ignored
2010-09-13, by blanchet
correctly thread parameter through
2010-09-13, by blanchet
indicate triviality in the list of proved things
2010-09-13, by blanchet
indicate which goals are trivial
2010-09-13, by blanchet
tuning
2010-09-13, by blanchet
tuning
2010-09-13, by blanchet
keep track of trivial vs. nontrivial calls using "try" for 30 seconds
2010-09-13, by blanchet
change signature of "Try.invoke_try" to make it more flexible
2010-09-13, by blanchet
use 30 s instead of 60 s as the default Sledgehammer timeout;
2010-09-13, by blanchet
no timeout for Auto Try, since the Auto Tools framework takes care of timeouts
2010-09-13, by blanchet
add Proof General option
2010-09-11, by blanchet
make Try's output more concise
2010-09-11, by blanchet
added Auto Try to the mix of automatic tools
2010-09-11, by blanchet
crank up Auto Tools timeout;
2010-09-11, by blanchet
make Auto Solve part of the "Auto Tools"
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
finished renaming "Auto_Counterexample" to "Auto_Tools"
2010-09-11, by blanchet
start renaming "Auto_Counterexample" to "Auto_Tools";
2010-09-11, by blanchet
setup Auto Sledgehammer
2010-09-11, by blanchet
make Mirabelle happy
2010-09-11, by blanchet
added Auto Sledgehammer docs
2010-09-11, by blanchet
change order of default ATPs;
2010-09-11, by blanchet
implemented Auto Sledgehammer
2010-09-11, by blanchet
document changes to Auto Nitpick
2010-09-11, by blanchet
change defaults of Auto Nitpick so that it consumes less resources (time and Kodkod threads)
2010-09-11, by blanchet
always handle type variables in typedefs as global
2010-09-11, by blanchet
removed duplicate lemma
2010-09-14, by nipkow
adding two more examples to example theory
2010-09-13, by bulwahn
handling function types more carefully than in e98a06145530
2010-09-13, by bulwahn
adding order on modes
2010-09-13, by bulwahn
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+1000
+3000
+10000
+30000
tip