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.
more "anti_sym" -> "antisym" (cf. a4179bf442d1);
2009-11-13, by wenzelm
merged
2009-11-13, by nipkow
renamed lemmas "anti_sym" -> "antisym"
2009-11-13, by nipkow
a few lemmas for point-free reasoning about transitive closure
2009-11-13, by krauss
merged
2009-11-13, by paulson
A number of theorems contributed by Jeremy Avigad
2009-11-13, by paulson
merged
2009-11-13, by bulwahn
merged
2009-11-12, by bulwahn
adding the predicate compiler quickcheck to the ex/ROOT.ML; adopting this quickcheck to the latest changes
2009-11-12, by bulwahn
removed annoying tracing message
2009-11-12, by bulwahn
added a tabled implementation of the reflexive transitive closure
2009-11-12, by bulwahn
merged
2009-11-12, by huffman
merged
2009-11-12, by huffman
improved ML interface to pcpodef
2009-11-12, by huffman
use Drule.standard (following typedef package), add pcpodef tactic interface
2009-11-11, by huffman
eliminated slightly odd (unused) "axiom" and "assumption" -- collapsed to unspecific "";
2009-11-12, by wenzelm
eliminated obsolete "internal" kind -- collapsed to unspecific "";
2009-11-12, by wenzelm
unused_thms: ignore kind -- already observes "concealed" flag;
2009-11-12, by wenzelm
all_valid_thms: more sophisticated check against global + local name space;
2009-11-12, by wenzelm
Remove map_compose, replaced by map_map
2009-11-12, by hoelzl
New list theorems; added map_map to simpset, this is the prefered direction; allow sorting by a key
2009-11-12, by hoelzl
Renamed upd_snd_conv to apsnd_conv to be consistent with apfst_conv; Added apsnd_apfst_commute
2009-11-12, by hoelzl
merged
2009-11-12, by haftmann
accomplish mutual recursion between fun and inst
2009-11-12, by haftmann
moved lemma map_of_zip_map to Map.thy
2009-11-12, by haftmann
merged
2009-11-12, by haftmann
explicit code lemmas produce nices code
2009-11-12, by haftmann
repaired broken code_const for term_of [String.literal]
2009-11-12, by haftmann
fixed soundness bug in Nitpick related to sets
2009-11-12, by blanchet
removed unnecessary oracle in the predicate compiler
2009-11-12, by bulwahn
improving code quality thanks to Florian's code review
2009-11-12, by bulwahn
renaming code_pred_intros to code_pred_intro
2009-11-12, by bulwahn
announcing the predicate compiler in NEWS and CONTRIBUTORS
2009-11-12, by bulwahn
new names for predicate functions in the predicate compiler
2009-11-12, by bulwahn
removed deprecated mode annotation parser; renamed accepted mode annotation parser to nicer naming
2009-11-12, by bulwahn
added another example to the predicate compiler
2009-11-12, by bulwahn
changed modes to expected_modes; added UNION to code_pred_inlining; fixed some examples; tuned
2009-11-12, by bulwahn
removed dummy setup for predicate compiler commands as the compiler is now part of HOL-Main
2009-11-12, by bulwahn
adopted predicate compiler examples to new syntax for modes
2009-11-12, by bulwahn
added interface of user proposals for names of generated constants
2009-11-12, by bulwahn
first steps towards a new mode datastructure; new syntax for mode annotations and new output of modes
2009-11-12, by bulwahn
adding more tests for the values command; adding some forbidden constants to inductify
2009-11-12, by bulwahn
Enables tests for locale functionality that is now available.
2009-11-11, by ballarin
merged
2009-11-11, by wenzelm
uniform use of simultabeous use_thys;
2009-11-11, by wenzelm
merged
2009-11-11, by haftmann
explicit invocation of code generation
2009-11-11, by haftmann
adding code equations for constructors
2009-11-11, by haftmann
tuned
2009-11-11, by haftmann
changed URL of SMT server,
2009-11-11, by boehmes
Added two new lemmas
2009-11-11, by paulson
tuned imports
2009-11-11, by haftmann
tuned
2009-11-11, by haftmann
local mutex for theory content/identity operations;
2009-11-11, by wenzelm
admit dummy implementation;
2009-11-11, by wenzelm
Toplevel.thread provides Isar-style exception output;
2009-11-10, by wenzelm
generalized Runtime.toplevel_error wrt. output function;
2009-11-10, by wenzelm
exported SimpleThread.attributes;
2009-11-10, by wenzelm
plain add_preference, no setmp_CRITICAL required;
2009-11-10, by wenzelm
adapted Theory_Data;
2009-11-10, by wenzelm
recovered update from 7264824baf66, which got lost in 7264824baf66;
2009-11-10, by wenzelm
merged
2009-11-10, by wenzelm
merged
2009-11-10, by haftmann
tuned header
2009-11-10, by haftmann
substantial simplification restores code generation
2009-11-10, by haftmann
lemmas about apfst and apsnd
2009-11-10, by haftmann
tuned imports
2009-11-10, by haftmann
merged
2009-11-10, by huffman
HOLCF example: domain package proofs done manually
2009-11-10, by huffman
add lemma parallel_fix_ind
2009-11-10, by huffman
add title/author block
2009-11-10, by huffman
theory of representable cpos
2009-11-10, by huffman
add map_map lemmas
2009-11-09, by huffman
add in_deflation relation, more lemmas about cast
2009-11-09, by huffman
ep_pair and deflation lemmas for powerdomain map functions
2009-11-09, by huffman
remove spurious parameter to "merge"
2009-11-10, by blanchet
merged, and renamed local "TheoryData" to "Data" (following common Isabelle conventions)
2009-11-10, by blanchet
fixed soundness bug in Nitpick related to sets of sets;
2009-11-10, by blanchet
added possibility to register datatypes as codatatypes in Nitpick;
2009-11-05, by blanchet
added datatype constructor cache in Nitpick (to speed up the scope enumeration) and never test more than 4096 scopes
2009-11-05, by blanchet
don't promise too much in the Nitpick manual
2009-11-05, by blanchet
merged
2009-11-05, by blanchet
added "nitpick_def" attribute to lfp/gfp definition generated by the inductive package;
2009-11-05, by blanchet
merged
2009-10-29, by blanchet
try very hard to remove temporary files generated by Nitpick in case of interruption
2009-10-29, by blanchet
eliminate two FIXMEs in Nitpick's monotonicity check code
2009-10-29, by blanchet
rename "NitpickMono" to "Nitpick_Mono" in example
2009-10-29, by blanchet
merged
2009-10-29, by blanchet
minor cleanup in Nitpick
2009-10-29, by blanchet
make "auto" SAT solver less verbose
2009-10-29, by blanchet
make "sizechange_tac" slightly less verbose
2009-10-29, by blanchet
don't run Nitpick at all if Kodkodi is not installed (as indicated by the $KODKODI variable)
2009-10-29, by blanchet
readded Predicate_Compile to Main
2009-10-29, by blanchet
merged
2009-10-29, by blanchet
fixed error in Nitpick's display of uncurried constants, which resulted in an exception
2009-10-29, by blanchet
fixed minor problems with Nitpick's documentation
2009-10-29, by blanchet
merged
2009-10-28, by blanchet
merged my Auto Nitpick change with Lukas's Predicate Compiler changes
2009-10-28, by blanchet
introduced Auto Nitpick in addition to Auto Quickcheck;
2009-10-28, by blanchet
use "get_goal" rather than "flat_goal" in Auto Quickcheck, since we don't need the extra facts for counterexample generation
2009-10-28, by blanchet
fix typo in Nitpick manual
2009-10-27, by blanchet
optimized Nitpick's encoding and rendering of datatypes whose constructors don't appear in the problem
2009-10-27, by blanchet
clean Nitpick's wellfoundedness cache once in a while, to avoid potential memory leak
2009-10-27, by blanchet
renamed Nitpick option "coalesce_type_vars" to "merge_type_vars" (shorter) and cleaned up old hacks that are no longer necessary
2009-10-27, by blanchet
eliminated some old uses of cumulative prems (!) in proof methods;
2009-11-10, by wenzelm
eliminated some unused/obsolete Args.bang_facts;
2009-11-10, by wenzelm
modernized structure Theory_Target;
2009-11-10, by wenzelm
removed unused Quickcheck_RecFun_Simps;
2009-11-10, by wenzelm
define simprocs: do not apply target_morphism prematurely, this is already done in LocalTheory.declaration;
2009-11-10, by wenzelm
bang_facts: legacy feature;
2009-11-10, by wenzelm
tuned proofs;
2009-11-10, by wenzelm
removed obsolete name_of -- cf. decode;
2009-11-10, by wenzelm
desymbolize: use Symbol.decode directly;
2009-11-10, by wenzelm
try SAT_Examples last, to minimize impact of global side-effects;
2009-11-10, by wenzelm
home-grown pretty printer for term -- Poly/ML 5.3.0 does not observe infix status of constructors (notably $);
2009-11-10, by wenzelm
Inserted missing theory dependency
2009-11-10, by paulson
merged
2009-11-09, by wenzelm
Merged.
2009-11-09, by ballarin
Removed obsolete code.
2009-11-09, by ballarin
updated to official Poly/ML 5.3.0;
2009-11-09, by wenzelm
switched some isatest sessions to official Poly/ML 5.3.0;
2009-11-09, by wenzelm
setup for official Poly/ML 5.3.0, which is now the default;
2009-11-09, by wenzelm
locale_const/target_notation: uniform use of Term.aconv_untyped;
2009-11-09, by wenzelm
eliminated hard tabulators;
2009-11-09, by wenzelm
fixed some inappropriate names
2009-11-09, by paulson
merged
2009-11-09, by paulson
New theory Probability/Borel.thy, and some associated lemmas
2009-11-09, by paulson
merged
2009-11-09, by haftmann
tuned error messages; tuned code
2009-11-09, by haftmann
follow standard theory merge behaviour: do not change already selected solver
2009-11-09, by boehmes
generalized proof by abstraction,
2009-11-09, by boehmes
made theory merge deterministic wrt. the selected solver
2009-11-09, by boehmes
merged
2009-11-08, by wenzelm
merged
2009-11-08, by berghofe
Repaired handling of comprehensions in "values" command.
2009-11-08, by berghofe
updated functor Theory_Data, Proof_Data, Generic_Data;
2009-11-08, by wenzelm
modernized structure Reorient_Proc;
2009-11-08, by wenzelm
adapted Theory_Data;
2009-11-08, by wenzelm
adapted Theory_Data;
2009-11-08, by wenzelm
tuned;
2009-11-08, by wenzelm
adapted Generic_Data, Proof_Data;
2009-11-08, by wenzelm
adapted Generic_Data;
2009-11-08, by wenzelm
modernized/simplified functor Theory_Data, Proof_Data, Generic_Data: eliminated Pretty.pp, discontinued mutable data;
2009-11-08, by wenzelm
added "declaration (pervasive)";
2009-11-08, by wenzelm
print_theorems: suppress concealed (global) facts, unless "!" option is given;
2009-11-08, by wenzelm
updated generated file;
2009-11-08, by wenzelm
modernized structure Random_Word;
2009-11-08, by wenzelm
init_component: slightly more robust read (raw input, succeed on non-terminated last line);
2009-11-08, by wenzelm
merged
2009-11-07, by webertj
Due to popular demand: added a function that benchmarks proof reconstruction
2009-11-07, by webertj
Turned sections into subsections (better document structure).
2009-11-07, by webertj
merged
2009-11-07, by huffman
merged
2009-11-07, by huffman
fix name of lemma snd_strict
2009-11-06, by huffman
use try instead of handle
2009-11-05, by huffman
map functions for various types, with ep_pair/deflation/finite_deflation lemmas
2009-11-05, by huffman
lemma deflation_strict
2009-11-05, by huffman
tuned ML_OPTIONS for SML/NJ -- for improved performance;
2009-11-07, by wenzelm
merged
2009-11-07, by haftmann
added predicate example
2009-11-07, by haftmann
tuned
2009-11-07, by haftmann
modernized primrec
2009-11-07, by haftmann
made SML/NJ happy
2009-11-06, by boehmes
merged
2009-11-06, by nipkow
merged
2009-11-04, by nipkow
Replaced exception CRing by error because it is meant for the user.
2009-10-29, by nipkow
merged
2009-11-06, by nipkow
Command atp_minimize uses the naive linear algorithm now
2009-11-06, by nipkow
merged
2009-11-06, by bulwahn
merged
2009-11-06, by bulwahn
merged
2009-11-06, by bulwahn
merge
2009-11-06, by bulwahn
merged
2009-11-06, by bulwahn
adopted the predicate compile quickcheck
2009-11-06, by bulwahn
made definition of functions generically for the different instances
2009-11-06, by bulwahn
renamed generator to random_function in the predicate compiler
2009-11-06, by bulwahn
improved handling of already defined functions in the predicate compiler; could cause trouble before when no modes for a predicate were infered
2009-11-06, by bulwahn
strictly respecting the line margin in the predicate compiler core
2009-11-06, by bulwahn
adopted mode syntax for values command
2009-11-06, by bulwahn
disabled upt example because of a problem due to overloaded constants with the predicate compiler
2009-11-06, by bulwahn
added optional mode annotations for parameters in the values command
2009-11-06, by bulwahn
moved values command from core to predicate compile
2009-11-06, by bulwahn
added further example of the values command
2009-11-06, by bulwahn
Adopted output of values command
2009-11-06, by bulwahn
improved handling of overloaded constants; examples with numerals
2009-11-06, by bulwahn
made SML/NJ happy; tuned
2009-11-06, by bulwahn
adding tracing function for evaluated code; annotated compilation in the predicate compiler
2009-11-06, by bulwahn
added documentation for local SMT solver setup and available SMT options,
2009-11-06, by boehmes
renamed method induct_scheme to induction_schema
2009-11-06, by krauss
NEWS
2009-11-06, by krauss
removed session SizeChange: outdated, only half-functional, alternatives exist (cf. size_change method)
2009-11-06, by krauss
renamed method sizechange to size_change
2009-11-06, by krauss
added boehmes and hoelzl to isatest mailings
2009-11-06, by krauss
merged
2009-11-06, by wenzelm
tuned
2009-11-06, by boehmes
Merged.
2009-11-05, by ballarin
Merged.
2009-11-04, by ballarin
Use PrintMode.setmp to make thread-safe; avoid code clones.
2009-11-04, by ballarin
Make output indenpendent of current print mode.
2009-11-02, by ballarin
Relax on type agreement with original context when applying term syntax.
2009-11-02, by ballarin
tuned;
2009-11-05, by wenzelm
proper naming convention lthy: local_theory, but ctxt: Proof.context for arbitrary context;
2009-11-05, by wenzelm
adapted LocalTheory.declaration;
2009-11-05, by wenzelm
allow "pervasive" local theory declarations, which are applied the background theory;
2009-11-05, by wenzelm
declare Spec_Rules for most basic definitional packages;
2009-11-05, by wenzelm
misc tuning and clarification;
2009-11-05, by wenzelm
scalable version of Named_Thms, using Item_Net;
2009-11-05, by wenzelm
merged
2009-11-05, by wenzelm
merged
2009-11-05, by wenzelm
more accurate cleanup;
2009-11-05, by wenzelm
merged
2009-11-05, by wenzelm
more accurate dependencies;
2009-11-05, by wenzelm
merged
2009-11-05, by boehmes
handle let expressions inside terms by unfolding (instead of raising an exception),
2009-11-05, by boehmes
shorter names for variables and verification conditions,
2009-11-05, by boehmes
added references to HOL-Boogie papers
2009-11-05, by boehmes
tuned header;
2009-11-05, by wenzelm
made SML/NJ happy;
2009-11-05, by wenzelm
eliminated funny record patterns and made SML/NJ happy;
2009-11-05, by wenzelm
proper header;
2009-11-05, by wenzelm
more accurate dependencies;
2009-11-05, by wenzelm
merged
2009-11-05, by wenzelm
added Tree23 to IsaMakefile
2009-11-04, by krauss
New
2009-11-04, by nipkow
merged
2009-11-04, by nipkow
fixed order of parameters in induction rules
2009-11-04, by nipkow
added bulwahn to isatest mailings
2009-11-04, by krauss
merged
2009-11-04, by nipkow
Completely overhauled
2009-11-04, by nipkow
better error handling for fixrec_simp
2009-11-03, by huffman
add more fixrec_simp rules
2009-11-03, by huffman
fixrec examples use fixrec_simp instead of fixpat
2009-11-03, by huffman
domain package registers fixrec_simp lemmas
2009-11-03, by huffman
merged
2009-11-03, by huffman
add fixrec_simp attribute and method (eventually to replace fixpat)
2009-11-03, by huffman
proper and unique case names for the split_vc method,
2009-11-03, by boehmes
merged
2009-11-03, by haftmann
merged
2009-11-03, by haftmann
always be qualified -- suspected smartness in fact never worked as expected
2009-11-03, by haftmann
pretty name for ==>
2009-11-03, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip