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.
dedicated exec ... syntax for open state monad (partly already introduces in d00a3f47b607)
2010-07-22, by haftmann
merged
2010-07-22, by wenzelm
more generous memory settings for scala check
2010-07-22, by haftmann
no polymorphic "var"s
2010-07-22, by blanchet
merged
2010-07-22, by bulwahn
adding checking of expected result for the tool quickcheck; annotated a few quickcheck examples
2010-07-21, by bulwahn
do a better job at Skolemizing in Nitpick, for TPTP FOF
2010-07-21, by blanchet
revert code that was submitted by mistake
2010-07-21, by blanchet
renamings + only need second component of name pool to reconstruct proofs
2010-07-21, by blanchet
rename "classrel" to "class_rel"
2010-07-21, by blanchet
rename "combtyp" constructors
2010-07-21, by blanchet
renamed "Literal" to "FOLLiteral"
2010-07-21, by blanchet
renamed "HOLClause" to "FOLClause" -- it's really a FOL clause with combinators
2010-07-21, by blanchet
merged
2010-07-21, by bulwahn
fixing quickcheck invocation in HOL-Mirabelle
2010-07-21, by bulwahn
hiding constants in Quickcheck_Types
2010-07-21, by bulwahn
adding a type for flat complete lattice to Quickcheck_Types
2010-07-21, by bulwahn
added new theories to IsaMakefile and ROOT.ML
2010-07-21, by bulwahn
adding Quickcheck examples for other quickcheck default types
2010-07-21, by bulwahn
adding Library theory for other quickcheck default types
2010-07-21, by bulwahn
removing obsolete ID in Quickcheck_Examples
2010-07-21, by bulwahn
correcting wellsortedness check and improving error message
2010-07-21, by bulwahn
using multiple default types in quickcheck
2010-07-21, by bulwahn
correcting merging of default_types
2010-07-21, by bulwahn
reordering quickcheck signature; exporting test_params and inspection function
2010-07-21, by bulwahn
changed default types to a list of types; extended quickcheck parameters to be a list of values to parse a list of default types
2010-07-21, by bulwahn
putting proof in the right context; adding if rewriting; tuned
2010-07-21, by bulwahn
load_thy: parallel parsing of units, which consist of statement/proof each;
2010-07-22, by wenzelm
eliminated some unreferenced identifiers;
2010-07-22, by wenzelm
tuned;
2010-07-22, by wenzelm
tuned comments;
2010-07-22, by wenzelm
replaced Source.of_list_limited by slightly more economic Source.of_string_limited;
2010-07-21, by wenzelm
deps_thy/load_thy: store compact text to reduce space by factor 12;
2010-07-21, by wenzelm
make SML/NJ happy, by adhoc type-constraints;
2010-07-21, by wenzelm
recovered benchmarks, which are not tested automatically;
2010-07-21, by wenzelm
made SML/NJ happy;
2010-07-21, by wenzelm
merged
2010-07-21, by wenzelm
abstract visualization of locale ingredients; all_locales yields proper locale identifiers
2010-07-21, by haftmann
tuned
2010-07-20, by haftmann
accomodate for scope of "as" binding in ML
2010-07-20, by haftmann
tuned code
2010-07-20, by haftmann
datatype classes are abstract
2010-07-20, by haftmann
avoid deprecation
2010-07-20, by haftmann
robustified metis proof
2010-07-20, by haftmann
modernized abel_cancel simproc setup
2010-07-19, by haftmann
keep explicit diff_def as legacy theorem; modernized abel_cancel simproc setup
2010-07-19, by haftmann
diff_eq_diff_less_eq' replaces diff_eq_diff_less_eq
2010-07-19, by haftmann
diff_minus subsumes diff_def
2010-07-19, by haftmann
tuned whitespace
2010-07-19, by haftmann
dropped essentially ineffective tuning
2010-07-19, by haftmann
discontinued pretending that abel_cancel is logic-independent; cleaned up junk
2010-07-19, by haftmann
merged
2010-07-19, by haftmann
merged
2010-07-19, by haftmann
distinguish different classes of const syntax
2010-07-19, by haftmann
Scala: subtle difference in printing strings vs. complex mixfix syntax
2010-07-19, by haftmann
check code generation for Scala
2010-07-19, by haftmann
dropped superfluous prefixes
2010-07-19, by haftmann
optional break
2010-07-19, by haftmann
consolidate const_syntax naming
2010-07-16, by haftmann
recovered benchmarks, which are not tested automatically;
2010-07-21, by wenzelm
reactivate SML/NJ test on macbroy28, while macbroy23 is unavailable;
2010-07-21, by wenzelm
eliminated old time_use/time_use_thy variants -- timing is implicitly controlled via Output.timing;
2010-07-21, by wenzelm
moved src/Tools/Compute_Oracle to src/HOL/Matrix/Compute_Oracle -- it actually depends on HOL anyway;
2010-07-21, by wenzelm
replaced Thy_Info.the_theory by Context.this_theory -- avoid referring to accidental theory loader state;
2010-07-21, by wenzelm
thm_deps/unused_thms: Context.get_theory based on proper theory ancestry, not accidental theory loader state;
2010-07-21, by wenzelm
explicit dependency on theory HOL;
2010-07-21, by wenzelm
ML antiquotations @{theory} and @{theory_ref} refer to the theory ancestry, not any accidental theory loader state;
2010-07-21, by wenzelm
added Context.get_theory -- avoid referring to accidental theory loader state (cf. Thy_Info.get_theory);
2010-07-21, by wenzelm
thy_deps: more direct comparison of sessions, which is presumably what "unfold" is meant to indicate here -- also avoid referring to accidental theory loader state;
2010-07-21, by wenzelm
clarified/exported Future.worker_subgroup, which is already the default for Future.fork;
2010-07-21, by wenzelm
qualified Thy_Info.get_theory;
2010-07-20, by wenzelm
discontinued pervasive val theory = Thy_Info.get_theory -- prefer antiquotations in most situations;
2010-07-20, by wenzelm
further Mac OS X deviations;
2010-07-20, by wenzelm
warning in proper transaction context;
2010-07-20, by wenzelm
SML/NJ: refrain from modifying toplevel pp for type string -- unclear if it could work here;
2010-07-20, by wenzelm
avoid duplicate printing of 'theory' state (cf. 173974e07dea);
2010-07-20, by wenzelm
toplevel pp for Proof.state and Toplevel.state;
2010-07-20, by wenzelm
execute document version at high priority;
2010-07-20, by wenzelm
Topelevel.run_command: interactive mode for initial 'theory' ensures that Thy_Info.begin_theory loads parent theories;
2010-07-20, by wenzelm
edit_document: join parent execution in synchronous/uninterruptible mode, to prevent spurious interrupts when cascaded executions run into each other;
2010-07-20, by wenzelm
back to more strict dependencies, even for canceled groups (reverting parts of 02936e77a07c);
2010-07-20, by wenzelm
export Graph.get_entry for convenience;
2010-07-20, by wenzelm
eliminated old-style sys_error/SYS_ERROR in favour of exception Fail -- after careful checking that there is no overlap with existing handling of that;
2010-07-20, by wenzelm
tuned;
2010-07-20, by wenzelm
observe follow_caret (again);
2010-07-20, by wenzelm
Session: predefined real time parameters;
2010-07-19, by wenzelm
bind and then latex symbols
2010-07-19, by haftmann
minor update of dependencies;
2010-07-18, by wenzelm
corrected range chec
2010-07-16, by haftmann
first roughly working version of Imperative HOL for Scala
2010-07-16, by haftmann
tuned
2010-07-16, by haftmann
merged
2010-07-16, by haftmann
a first sketch for Imperative HOL witht Scala
2010-07-16, by haftmann
don't fail gracefully
2010-07-16, by haftmann
restored long-broken syntax sanity checks
2010-07-16, by haftmann
tuned interpunctation
2010-07-16, by haftmann
fragments of Scala
2010-07-16, by haftmann
merged
2010-07-15, by haftmann
adjusted; fixed typo
2010-07-15, by haftmann
dropped spurious export_code
2010-07-15, by haftmann
use different log server (macbroy23 down)
2010-07-14, by kleing
more consistent spacing in generated monadic code
2010-07-14, by haftmann
braced needed in layout-insensitive syntax
2010-07-14, by haftmann
repaired some implementations of imperative operations
2010-07-14, by haftmann
repaired reference implementation for OCaml
2010-07-14, by haftmann
part of pervasive test
2010-07-14, by haftmann
avoid ambiguities; tuned
2010-07-14, by haftmann
repaired of_list implementation for SML, OCaml
2010-07-14, by haftmann
avoid export_code ... file -
2010-07-14, by haftmann
explicit optional checking
2010-07-14, by haftmann
added Isar syntax for code checking
2010-07-14, by haftmann
corrected import
2010-07-14, by haftmann
use generic description slot for formal code checking
2010-07-14, by haftmann
formal slot for code checker
2010-07-14, by haftmann
export_code without file prints to standard output
2010-07-14, by haftmann
check without explicit path
2010-07-14, by haftmann
load cache_io before code generator; moved adhoc-overloading to generic tools
2010-07-14, by haftmann
tuned infix syntax
2010-07-14, by haftmann
dropped M suffix; added predicate monad bind
2010-07-14, by haftmann
self-built symbol for part of bind operator
2010-07-14, by haftmann
redirect stderr to stdout
2010-07-14, by haftmann
merged
2010-07-13, by paulson
merged
2010-07-13, by paulson
corrected mixfix declarations and tidied proofs
2010-07-13, by paulson
merged
2010-07-13, by paulson
Fixed syntax and tidied some proofs
2010-07-13, by paulson
correcting function name of generator for products of traditional code generator (introduced in 0040bafffdef)
2010-07-13, by bulwahn
consolidated names of theorems
2010-07-13, by haftmann
qualified names for (really) all array operations
2010-07-13, by haftmann
canonical argument order for get
2010-07-13, by haftmann
qualified names for (almost) all array operations
2010-07-13, by haftmann
canonical argument order for present
2010-07-13, by haftmann
canonical argument order for length
2010-07-13, by haftmann
merged
2010-07-13, by kleing
new crontab
2010-07-13, by kleing
merged
2010-07-13, by haftmann
proper merge of operation changes and generic do-syntax
2010-07-13, by haftmann
merged
2010-07-13, by haftmann
hide_const; update replaces change
2010-07-13, by haftmann
remove separate afp settings again, use plain mac-poly64-M4 instead.
2010-07-13, by kleing
merged
2010-07-13, by kleing
new settings for afp test
2010-07-13, by kleing
Heap_Monad uses Monad_Syntax
2010-07-13, by krauss
State_Monad uses Monad_Syntax
2010-07-13, by krauss
uniform do notation for monads
2010-07-13, by krauss
generic ad-hoc overloading via check/uncheck
2010-07-13, by krauss
corrected title
2010-07-13, by haftmann
theorem collections do not contain default rules any longer
2010-07-13, by haftmann
fixed handling of Ball/Bex: turn equalities into meta-equalities for the rewriting conversions;
2010-07-13, by boehmes
removed unused/untested IOA 'automaton' package;
2010-07-12, by wenzelm
removed impractical tolerate_legacy_features flag;
2010-07-12, by wenzelm
tuned comment;
2010-07-12, by wenzelm
removed legacy aliases;
2010-07-12, by wenzelm
moved misc legacy stuff from OldGoals to Misc_Legacy;
2010-07-12, by wenzelm
eliminated OldGoals.strip_context;
2010-07-12, by wenzelm
removed old HOL/HOLCF-Modelcheck setup, which has been unused/untested for many years;
2010-07-12, by wenzelm
do not intercept ML exceptions -- printing exception positions/text is the job of the Isar/ML toplevel;
2010-07-12, by wenzelm
some modernization of really ancient Meson experiments;
2010-07-12, by wenzelm
dropped empty theory
2010-07-12, by haftmann
moved auxiliary lemma
2010-07-12, by haftmann
dropped unused lemmas of dubious value
2010-07-12, by haftmann
dropped unused lemmas of dubious value
2010-07-12, by haftmann
split off mrec into separate theory
2010-07-12, by haftmann
spelt out relational framework in a consistent way
2010-07-12, by haftmann
avoid explicit mandatory prefix markers when prefixes are mandatory implicitly
2010-07-12, by haftmann
merged
2010-07-12, by haftmann
moved co-regularity to class section; avoid duplicated class_deps
2010-07-12, by haftmann
dropped superfluous [code del]s
2010-07-12, by haftmann
merged
2010-07-12, by haftmann
dropped superfluous [code del]s
2010-07-12, by haftmann
more regular session structure
2010-07-12, by haftmann
regular image setup for HOL-Library (cf. 4915de09b4d3 and ccae4ecd67f4) -- note that document preparation requires a separate session directory, and library.ML is a bit too generic as a file in the default load path;
2010-07-10, by wenzelm
merged
2010-07-10, by wenzelm
Added current crontab of macbroy28
2010-07-09, by kleing
moved example to its own file in HOL/ex
2010-07-09, by krauss
merged
2010-07-09, by haftmann
pervasive success combinator
2010-07-09, by haftmann
added "while_option", which needs no well-foundedness; defined "while" in terms of "while_option"
2010-07-09, by krauss
avoid slightly odd "M" suffix; rename mapM to fold_map (fold_map_abort would be more correct, though)
2010-07-09, by haftmann
adapted to changes
2010-07-09, by haftmann
guard combinator
2010-07-09, by haftmann
tuned reference theory
2010-07-09, by haftmann
tuned array theory
2010-07-09, by haftmann
nicer xsymbol syntax for fcomp and scomp
2010-07-09, by haftmann
dropped ancient in-place compilation of SML; more tests
2010-07-08, by haftmann
updated documentation
2010-07-08, by haftmann
dropped ancient in-place compilation of SML
2010-07-08, by haftmann
more accurate dependencies
2010-07-08, by haftmann
empty default
2010-07-08, by haftmann
checking generated code for various target languages
2010-07-08, by haftmann
tuned titles
2010-07-08, by haftmann
tuned module names
2010-07-08, by haftmann
tuned tabs
2010-07-08, by haftmann
tuned script
2010-07-08, by haftmann
combinator with_tmp_dir
2010-07-08, by haftmann
rm_tree: remove entire file system trees
2010-07-08, by haftmann
Boxes may now have different widths.
2010-07-07, by berghofe
tuned
2010-07-07, by hoelzl
replaced manual derivation of equations for inductive predicates by automatic derivation by inductive_simps
2010-07-07, by bulwahn
added NEWS entry
2010-07-07, by bulwahn
added the new command inductive_cases to derive simplification equations for inductive predicates; added binding simps for general simplification equation
2010-07-07, by bulwahn
merged
2010-07-06, by huffman
generalize type of is_interval to class euclidean_space
2010-07-05, by huffman
section -> subsection
2010-07-05, by huffman
generalize some lemmas about derivatives
2010-07-04, by huffman
uniqueness of Frechet derivative
2010-07-04, by huffman
implode pseudo utf8, i.e. decode byte-stuffed low ASCII characters;
2010-07-06, by wenzelm
merged
2010-07-06, by wenzelm
even more fun with primrec
2010-07-06, by haftmann
refactored reference operations
2010-07-06, by haftmann
tuned
2010-07-06, by haftmann
tuned empty heap
2010-07-06, by haftmann
merged
2010-07-05, by paulson
merged
2010-07-05, by paulson
Unification (flexflex) bug fix; making "auto" deterministic
2010-07-05, by paulson
moved "open" operations from Heap.thy to Array.thy and Ref.thy
2010-07-05, by haftmann
only definite assignment
2010-07-05, by haftmann
moved special operation array_ran here
2010-07-05, by haftmann
remove primitive operation Heap.array in favour of Heap.array_of_list
2010-07-05, by haftmann
tuned proof
2010-07-05, by haftmann
tuned
2010-07-05, by haftmann
Outer_Syntax.prepare_command: disallow control commands here, and consequently in Isar documents;
2010-07-05, by wenzelm
specific ML_val vs. ML_command;
2010-07-05, by wenzelm
async_state: report within proper transaction context;
2010-07-05, by wenzelm
merged
2010-07-05, by haftmann
simplified representation of monad type
2010-07-05, by haftmann
attempt to reconstruct missing HOL/Codegenerator_Test/ROOT.ML;
2010-07-05, by wenzelm
merged
2010-07-05, by wenzelm
updated document
2010-07-05, by haftmann
dropped passed irregular names
2010-07-05, by haftmann
adapt Nitpick to "prod_case" and "*" -> "sum" renaming;
2010-07-03, by blanchet
remove needless signature entry
2010-07-03, by blanchet
references to ghc and ocaml
2010-07-02, by haftmann
explicit code_datatype declaration prevents multiple instantiations later on
2010-07-02, by haftmann
refrain from using datatype declaration -- opens chance for quickcheck later on
2010-07-02, by haftmann
tuned proof
2010-07-02, by haftmann
reverted to verion from fc27be4c6b1c
2010-07-02, by haftmann
traceback for error messages
2010-07-02, by haftmann
accomodate for different behvaiour of nitpick (c.f. also 180e80b4eac1)
2010-07-02, by haftmann
introduced distinct session HOL-Codegenerator_Test
2010-07-02, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip