Fri, 27 Sep 2013 15:38:23 +0200 |
nipkow |
added code eqns for bounded LEAST operator
|
file |
diff |
annotate
|
Thu, 26 Sep 2013 13:37:33 +0200 |
lammich |
Added symmetric code_unfold-lemmas for null and is_none
|
file |
diff |
annotate
|
Wed, 18 Sep 2013 18:11:32 +0200 |
traytel |
added two functions to List (one contributed by Manuel Eberl)
|
file |
diff |
annotate
|
Wed, 18 Sep 2013 12:16:10 +0200 |
nipkow |
added and tuned lemmas
|
file |
diff |
annotate
|
Thu, 05 Sep 2013 11:10:51 +0200 |
traytel |
list_to_set_comprehension: don't crash in case distinctions on datatypes with even number of constructors
|
file |
diff |
annotate
|
Tue, 03 Sep 2013 01:12:40 +0200 |
wenzelm |
tuned proofs -- clarified flow of facts wrt. calculation;
|
file |
diff |
annotate
|
Tue, 13 Aug 2013 17:45:22 +0200 |
wenzelm |
merged
|
file |
diff |
annotate
|
Tue, 13 Aug 2013 16:25:47 +0200 |
wenzelm |
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
|
file |
diff |
annotate
|
Tue, 13 Aug 2013 15:59:22 +0200 |
kuncar |
move Lifting/Transfer relevant parts of Library/Quotient_* to Main
|
file |
diff |
annotate
|
Sun, 23 Jun 2013 21:16:07 +0200 |
haftmann |
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
|
file |
diff |
annotate
|
Sat, 15 Jun 2013 17:19:23 +0200 |
haftmann |
lifting for primitive definitions;
|
file |
diff |
annotate
|
Sat, 15 Jun 2013 17:19:23 +0200 |
haftmann |
selection operator smallest_prime_beyond
|
file |
diff |
annotate
|
Sat, 25 May 2013 18:30:38 +0200 |
wenzelm |
merged
|
file |
diff |
annotate
|
Sat, 25 May 2013 15:37:53 +0200 |
wenzelm |
syntax translations always depend on context;
|
file |
diff |
annotate
|
Sat, 25 May 2013 15:44:29 +0200 |
haftmann |
weaker precendence of syntax for big intersection and union on sets
|
file |
diff |
annotate
|
Fri, 24 May 2013 17:00:46 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Thu, 23 May 2013 14:22:49 +0200 |
noschinl |
more lemmas for sorted_list_of_set
|
file |
diff |
annotate
|
Mon, 06 May 2013 02:48:18 +0200 |
nipkow |
tail recursive version of map, for code generation, optionally
|
file |
diff |
annotate
|
Tue, 23 Apr 2013 11:14:51 +0200 |
haftmann |
tuned: unnamed contexts, interpretation and sublocale in locale target;
|
file |
diff |
annotate
|
Thu, 18 Apr 2013 17:07:01 +0200 |
wenzelm |
simplifier uses proper Proof.context instead of historic type simpset;
|
file |
diff |
annotate
|
Fri, 05 Apr 2013 22:08:42 +0200 |
traytel |
allow redundant cases in the list comprehension translation
|
file |
diff |
annotate
|
Tue, 22 Jan 2013 14:33:45 +0100 |
traytel |
separate data used for case translation from the datatype package
|
file |
diff |
annotate
|
Tue, 22 Jan 2013 13:32:41 +0100 |
berghofe |
case translations performed in a separate check phase (with adjustments by traytel)
|
file |
diff |
annotate
|
Wed, 27 Mar 2013 10:55:05 +0100 |
haftmann |
centralized various multiset operations in theory multiset;
|
file |
diff |
annotate
|
Tue, 26 Mar 2013 20:49:57 +0100 |
haftmann |
explicit sublocale dependency for Min/Max yields more appropriate Min/Max prefix for a couple of facts
|
file |
diff |
annotate
|
Sat, 23 Mar 2013 20:50:39 +0100 |
haftmann |
fundamental revision of big operators on sets
|
file |
diff |
annotate
|
Thu, 28 Feb 2013 17:14:55 +0100 |
wenzelm |
provide common HOLogic.conj_conv and HOLogic.eq_conv;
|
file |
diff |
annotate
|
Thu, 28 Feb 2013 16:54:52 +0100 |
wenzelm |
just one HOLogic.Trueprop_conv, with regular exception CTERM;
|
file |
diff |
annotate
|
Mon, 25 Feb 2013 12:17:50 +0100 |
wenzelm |
prefer stateless 'ML_val' for tests;
|
file |
diff |
annotate
|
Sun, 17 Feb 2013 21:29:30 +0100 |
haftmann |
Sieve of Eratosthenes
|
file |
diff |
annotate
|
Sun, 17 Feb 2013 11:34:40 +0100 |
haftmann |
simplified construction of upto_aux
|
file |
diff |
annotate
|
Sat, 16 Feb 2013 15:27:10 +0100 |
nipkow |
tail recursive code for function "upto"
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 11:47:33 +0100 |
haftmann |
systematic conversions between nat and nibble/char;
|
file |
diff |
annotate
|
Thu, 14 Feb 2013 12:24:42 +0100 |
haftmann |
abandoned theory Plain
|
file |
diff |
annotate
|
Wed, 13 Feb 2013 13:38:52 +0100 |
haftmann |
combinator List.those;
|
file |
diff |
annotate
|
Fri, 14 Dec 2012 19:51:20 +0100 |
nipkow |
unified layout of defs
|
file |
diff |
annotate
|
Fri, 07 Dec 2012 16:25:33 +0100 |
wenzelm |
avoid ML_file in large theory files to improve performance of dependency discovery of main HOL (approx. 1s CPU time) -- relevant for any application using it, e.g. small paper sessions;
|
file |
diff |
annotate
|
Tue, 20 Nov 2012 18:59:35 +0100 |
hoelzl |
add Countable_Set theory
|
file |
diff |
annotate
|
Thu, 08 Nov 2012 11:59:48 +0100 |
bulwahn |
adjusting proofs as the set_comprehension_pointfree simproc breaks some existing proofs
|
file |
diff |
annotate
|
Sun, 21 Oct 2012 17:04:13 +0200 |
webertj |
merged
|
file |
diff |
annotate
|
Fri, 19 Oct 2012 15:12:52 +0200 |
webertj |
Renamed {left,right}_distrib to distrib_{right,left}.
|
file |
diff |
annotate
|
Sat, 20 Oct 2012 09:12:16 +0200 |
haftmann |
moved quite generic material from theory Enum to more appropriate places
|
file |
diff |
annotate
|
Wed, 10 Oct 2012 15:16:44 +0200 |
Andreas Lochbihler |
tail-recursive implementation for length
|
file |
diff |
annotate
|
Tue, 09 Oct 2012 16:57:58 +0200 |
kuncar |
rename Set.project to Set.filter - more appropriate name
|
file |
diff |
annotate
|
Mon, 08 Oct 2012 12:03:49 +0200 |
haftmann |
consolidated names of theorems on composition;
|
file |
diff |
annotate
|
Wed, 22 Aug 2012 22:55:41 +0200 |
wenzelm |
prefer ML_file over old uses;
|
file |
diff |
annotate
|
Thu, 16 Aug 2012 14:07:32 +0200 |
haftmann |
prefer eta-expanded code equations for fold, to accomodate tail recursion optimisation in Scala
|
file |
diff |
annotate
|
Tue, 31 Jul 2012 13:55:39 +0200 |
kuncar |
more set operations expressed by Finite_Set.fold
|
file |
diff |
annotate
|
Mon, 30 Apr 2012 12:14:53 +0200 |
bulwahn |
making sorted_list_of_set executable
|
file |
diff |
annotate
|
Sat, 21 Apr 2012 06:49:04 +0200 |
huffman |
strengthen rule list_all2_induct
|
file |
diff |
annotate
|
Thu, 12 Apr 2012 11:01:15 +0200 |
bulwahn |
merged
|
file |
diff |
annotate
|
Tue, 03 Apr 2012 17:26:30 +0900 |
griff |
renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")
|
file |
diff |
annotate
|
Fri, 06 Apr 2012 19:23:51 +0200 |
haftmann |
abandoned almost redundant *_foldr lemmas
|
file |
diff |
annotate
|
Fri, 06 Apr 2012 19:18:00 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
Fri, 06 Apr 2012 18:17:16 +0200 |
haftmann |
no preference wrt. fold(l/r); prefer fold rather than foldr for iterating over lists in generated code
|
file |
diff |
annotate
|
Mon, 26 Mar 2012 21:00:23 +0200 |
nipkow |
reverted to canonical name
|
file |
diff |
annotate
|
Mon, 26 Mar 2012 18:54:41 +0200 |
nipkow |
Functions and lemmas by Christian Sternagel
|
file |
diff |
annotate
|
Sun, 25 Mar 2012 20:15:39 +0200 |
huffman |
merged fork with new numeral representation (see NEWS)
|
file |
diff |
annotate
|
Tue, 13 Mar 2012 13:31:26 +0100 |
wenzelm |
tuned proofs -- eliminated pointless chaining of facts after 'interpret';
|
file |
diff |
annotate
|
Mon, 12 Mar 2012 21:41:11 +0100 |
noschinl |
tuned proofs
|
file |
diff |
annotate
|