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
|
Mon, 27 Feb 2012 09:01:49 +0100 |
nipkow |
converting "set [...]" to "{...}" in evaluation results
|
file |
diff |
annotate
|
Sat, 25 Feb 2012 09:07:37 +0100 |
bulwahn |
one general list_all2_update_cong instead of two special ones
|
file |
diff |
annotate
|
Fri, 24 Feb 2012 22:46:44 +0100 |
haftmann |
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
|
file |
diff |
annotate
|
Fri, 24 Feb 2012 09:40:02 +0100 |
haftmann |
given up disfruitful branch
|
file |
diff |
annotate
|
Thu, 23 Feb 2012 21:25:59 +0100 |
haftmann |
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
|
file |
diff |
annotate
|
Thu, 16 Feb 2012 09:18:23 +0100 |
bulwahn |
removing unnecessary premises in theorems of List theory
|
file |
diff |
annotate
|
Fri, 10 Feb 2012 09:47:59 +0100 |
Cezary Kaliszyk |
more specification of the quotient package in IsarRef
|
file |
diff |
annotate
|
Wed, 08 Feb 2012 01:49:33 +0100 |
blanchet |
use 'primrec' to define "rotate1", for uniformity (and to help first-order tools that rely on "Spec_Rules")
|
file |
diff |
annotate
|
Wed, 08 Feb 2012 00:55:06 +0100 |
blanchet |
removed fact that confuses SPASS -- better rely on "rev_rev_ident", which is stronger and more ATP friendly
|
file |
diff |
annotate
|
Sun, 05 Feb 2012 10:43:52 +0100 |
bulwahn |
adding code equation for Relation.image; adding map_project as correspondence to map_filter on lists
|
file |
diff |
annotate
|
Sun, 05 Feb 2012 08:24:39 +0100 |
bulwahn |
another try to improve code generation of set equality (cf. da32cf32c0c7)
|
file |
diff |
annotate
|
Thu, 02 Feb 2012 10:12:30 +0100 |
bulwahn |
adding a minimally refined equality on sets for code generation
|
file |
diff |
annotate
|
Tue, 31 Jan 2012 15:39:45 +0100 |
bulwahn |
adding code equation for setsum
|
file |
diff |
annotate
|
Mon, 23 Jan 2012 17:29:19 +0100 |
huffman |
generalize type of List.listrel
|
file |
diff |
annotate
|
Mon, 23 Jan 2012 14:07:36 +0100 |
bulwahn |
adding code generation for some list relations
|
file |
diff |
annotate
|
Tue, 10 Jan 2012 18:12:03 +0100 |
berghofe |
pred_subset/equals_eq are now standard pred_set_conv rules
|
file |
diff |
annotate
|
Sat, 07 Jan 2012 20:44:23 +0100 |
haftmann |
massaging of code setup for sets
|
file |
diff |
annotate
|
Sat, 07 Jan 2012 11:45:53 +0100 |
haftmann |
corrected slip
|
file |
diff |
annotate
|
Sat, 07 Jan 2012 09:32:01 +0100 |
haftmann |
restore convenient code_abbrev declarations (particulary important if List.set is not the formal constructor for sets)
|
file |
diff |
annotate
|
Fri, 06 Jan 2012 22:16:01 +0100 |
haftmann |
moved lemmas about List.set and set operations to List theory
|
file |
diff |
annotate
|
Fri, 06 Jan 2012 20:39:50 +0100 |
haftmann |
farewell to theory More_List
|
file |
diff |
annotate
|
Fri, 06 Jan 2012 17:44:42 +0100 |
wenzelm |
improved list comprehension syntax: more careful treatment of position constraints, which enables PIDE markup;
|
file |
diff |
annotate
|
Fri, 06 Jan 2012 10:19:49 +0100 |
haftmann |
incorporated canonical fold combinator on lists into body of List theory; refactored passages on List.fold(l/r)
|
file |
diff |
annotate
|
Thu, 05 Jan 2012 18:18:39 +0100 |
wenzelm |
improved case syntax: more careful treatment of position constraints, which enables PIDE markup;
|
file |
diff |
annotate
|
Thu, 29 Dec 2011 13:42:21 +0100 |
haftmann |
qualified Finite_Set.fold
|
file |
diff |
annotate
|
Thu, 29 Dec 2011 10:47:55 +0100 |
haftmann |
attribute code_abbrev superseedes code_unfold_post; tuned text
|
file |
diff |
annotate
|
Tue, 27 Dec 2011 09:15:26 +0100 |
haftmann |
dropped fact whose names clash with corresponding facts on canonical fold
|
file |
diff |
annotate
|
Sat, 24 Dec 2011 15:53:10 +0100 |
haftmann |
dropped obsolete lemma member_set
|
file |
diff |
annotate
|
Mon, 19 Dec 2011 14:41:08 +0100 |
noschinl |
add lemmas
|
file |
diff |
annotate
|
Thu, 15 Dec 2011 18:08:40 +0100 |
wenzelm |
clarified module dependencies: Datatype_Data, Datatype_Case, Rep_Datatype;
|
file |
diff |
annotate
|
Tue, 13 Dec 2011 22:44:16 +0100 |
noschinl |
added lemmas
|
file |
diff |
annotate
|
Fri, 09 Dec 2011 13:42:16 +0100 |
huffman |
add induction rule for list_all2
|
file |
diff |
annotate
|
Thu, 08 Dec 2011 13:53:27 +0100 |
bulwahn |
removing special code generator setup for hd and last function because this causes problems with quickcheck narrowing as the Haskell Prelude functions throw errors that cannot be caught instead of PatternFail exceptions
|
file |
diff |
annotate
|
Thu, 01 Dec 2011 15:41:58 +0100 |
hoelzl |
cardinality of sets of lists
|
file |
diff |
annotate
|
Sun, 20 Nov 2011 21:07:10 +0100 |
wenzelm |
eliminated obsolete "standard";
|
file |
diff |
annotate
|
Wed, 19 Oct 2011 08:37:27 +0200 |
bulwahn |
removing old code generator setup for lists
|
file |
diff |
annotate
|
Mon, 03 Oct 2011 14:43:12 +0200 |
bulwahn |
adding lemma to List library for executable equation of the (refl) transitive closure
|
file |
diff |
annotate
|
Wed, 14 Sep 2011 10:08:52 -0400 |
hoelzl |
renamed Complete_Lattices lemmas, removed legacy names
|
file |
diff |
annotate
|
Tue, 13 Sep 2011 17:07:33 -0700 |
huffman |
tuned proofs
|
file |
diff |
annotate
|
Tue, 13 Sep 2011 12:14:29 +0200 |
bulwahn |
added lemma motivated by a more specific lemma in the AFP-KBPs theories
|
file |
diff |
annotate
|
Mon, 12 Sep 2011 07:55:43 +0200 |
nipkow |
new fastforce replacing fastsimp - less confusing name
|
file |
diff |
annotate
|
Thu, 01 Sep 2011 13:18:27 +0200 |
blanchet |
added two lemmas about "distinct" to help Sledgehammer
|
file |
diff |
annotate
|
Tue, 30 Aug 2011 20:10:48 +0200 |
bulwahn |
adding list_size_append (thanks to Rene Thiemann)
|
file |
diff |
annotate
|
Tue, 30 Aug 2011 20:10:47 +0200 |
bulwahn |
strengthening list_size_pointwise (thanks to Rene Thiemann)
|
file |
diff |
annotate
|
Fri, 26 Aug 2011 11:22:47 +0200 |
nipkow |
added lemma
|
file |
diff |
annotate
|
Tue, 02 Aug 2011 10:36:50 +0200 |
krauss |
moved recdef package to HOL/Library/Old_Recdef.thy
|
file |
diff |
annotate
|
Wed, 29 Jun 2011 17:35:46 +0200 |
wenzelm |
modernized some simproc setup;
|
file |
diff |
annotate
|
Mon, 27 Jun 2011 17:04:04 +0200 |
krauss |
new Datatype.info_of_constr with strict behaviour wrt. to overloaded constructors -- side effect: function package correctly identifies 0::int as a non-constructor;
|
file |
diff |
annotate
|
Thu, 09 Jun 2011 16:34:49 +0200 |
wenzelm |
discontinued Name.variant to emphasize that this is old-style / indirect;
|
file |
diff |
annotate
|
Fri, 20 May 2011 11:44:16 +0200 |
haftmann |
names of fold_set locales resemble name of characteristic property more closely
|
file |
diff |
annotate
|
Sat, 14 May 2011 18:26:25 +0200 |
haftmann |
use pointfree characterisation for fold_set locale
|
file |
diff |
annotate
|
Mon, 09 May 2011 16:11:20 +0200 |
noschinl |
add a lemma about commutative append to List.thy
|
file |
diff |
annotate
|
Mon, 09 May 2011 12:26:25 +0200 |
noschinl |
removed assumption from lemma List.take_add
|
file |
diff |
annotate
|
Tue, 19 Apr 2011 23:57:28 +0200 |
wenzelm |
eliminated Codegen.mode in favour of explicit argument;
|
file |
diff |
annotate
|
Sat, 16 Apr 2011 16:15:37 +0200 |
wenzelm |
modernized structure Proof_Context;
|
file |
diff |
annotate
|
Sat, 16 Apr 2011 15:25:25 +0200 |
wenzelm |
prefer local name spaces;
|
file |
diff |
annotate
|
Wed, 06 Apr 2011 23:04:00 +0200 |
wenzelm |
separate structure Term_Position;
|
file |
diff |
annotate
|
Wed, 30 Mar 2011 20:19:21 +0200 |
wenzelm |
actually check list comprehension examples;
|
file |
diff |
annotate
|
Mon, 28 Mar 2011 23:49:53 +0200 |
wenzelm |
list comprehension: strip positions where the translation cannot handle them right now;
|
file |
diff |
annotate
|
Tue, 22 Mar 2011 20:44:47 +0100 |
wenzelm |
more selective strip_positions in case patterns -- reactivate translations based on "case _ of _" in HOL and special patterns in HOLCF;
|
file |
diff |
annotate
|
Tue, 15 Mar 2011 22:04:02 +0100 |
nipkow |
added lemma
|
file |
diff |
annotate
|
Fri, 25 Feb 2011 14:25:41 +0100 |
nipkow |
added simp lemma nth_Cons_pos to List
|
file |
diff |
annotate
|
Thu, 03 Feb 2011 18:57:42 +0100 |
wenzelm |
explicit is better than implicit;
|
file |
diff |
annotate
|
Tue, 11 Jan 2011 14:12:37 +0100 |
haftmann |
"enriched_type" replaces less specific "type_lifting"
|
file |
diff |
annotate
|
Fri, 07 Jan 2011 18:10:35 +0100 |
bulwahn |
adding simproc to rewrite list comprehensions to set comprehensions; adopting proofs
|
file |
diff |
annotate
|
Tue, 21 Dec 2010 17:52:23 +0100 |
haftmann |
tuned type_lifting declarations
|
file |
diff |
annotate
|
Fri, 17 Dec 2010 17:43:54 +0100 |
wenzelm |
replaced command 'nonterminals' by slightly modernized version 'nonterminal';
|
file |
diff |
annotate
|
Wed, 08 Dec 2010 13:34:50 +0100 |
haftmann |
primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`
|
file |
diff |
annotate
|
Mon, 06 Dec 2010 09:19:10 +0100 |
haftmann |
replace `type_mapper` by the more adequate `type_lifting`
|
file |
diff |
annotate
|
Sun, 28 Nov 2010 15:20:51 +0100 |
nipkow |
gave more standard finite set rules simp and intro attribute
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 11:34:58 +0100 |
bulwahn |
adding code equations for EX1 on finite types
|
file |
diff |
annotate
|
Thu, 18 Nov 2010 17:01:16 +0100 |
haftmann |
mapper for list type; map_pair replaces prod_fun
|
file |
diff |
annotate
|
Wed, 17 Nov 2010 21:35:23 +0100 |
nipkow |
code eqn for slice was missing; redefined splice with fun
|
file |
diff |
annotate
|
Fri, 05 Nov 2010 08:16:34 +0100 |
bulwahn |
added two lemmas about injectivity of concat to the list theory
|
file |
diff |
annotate
|
Tue, 02 Nov 2010 16:31:57 +0100 |
haftmann |
lemmas sorted_map_same, sorted_same
|
file |
diff |
annotate
|
Thu, 28 Oct 2010 17:54:09 +0200 |
nipkow |
added lemmas about listrel(1)
|
file |
diff |
annotate
|
Wed, 27 Oct 2010 16:40:31 +0200 |
haftmann |
sorting: avoid _key suffix if lemma applies both to simple and generalized variant; generalized insort_insert to insort_insert_key; additional lemmas
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 16:39:21 +0200 |
haftmann |
include ATP in theory List -- avoid theory edge by-passing the prominent list theory
|
file |
diff |
annotate
|
Mon, 25 Oct 2010 13:34:58 +0200 |
haftmann |
dropped (almost) redundant distinct.induct rule; distinct_simps again named distinct.simps
|
file |
diff |
annotate
|
Sun, 24 Oct 2010 20:19:00 +0200 |
nipkow |
nat_number -> eval_nat_numeral
|
file |
diff |
annotate
|
Wed, 06 Oct 2010 17:44:21 +0200 |
blanchet |
merged
|
file |
diff |
annotate
|
Mon, 04 Oct 2010 22:45:09 +0200 |
blanchet |
move Metis into Plain
|
file |
diff |
annotate
|
Mon, 04 Oct 2010 12:22:58 +0200 |
haftmann |
turned distinct and sorted into inductive predicates: yields nice induction principles for free; more elegant proofs
|
file |
diff |
annotate
|
Tue, 28 Sep 2010 15:21:45 +0200 |
haftmann |
localized listsum
|
file |
diff |
annotate
|
Mon, 27 Sep 2010 14:13:22 +0200 |
haftmann |
lemma remdups_map_remdups
|
file |
diff |
annotate
|
Wed, 22 Sep 2010 16:52:09 +0200 |
nipkow |
more lists lemmas
|
file |
diff |
annotate
|
Tue, 21 Sep 2010 02:03:40 +0200 |
nipkow |
new lemma
|
file |
diff |
annotate
|
Fri, 17 Sep 2010 20:53:50 +0200 |
haftmann |
generalized lemma insort_remove1 to insort_key_remove1
|
file |
diff |
annotate
|
Mon, 13 Sep 2010 11:13:15 +0200 |
nipkow |
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
|
file |
diff |
annotate
|
Fri, 10 Sep 2010 10:21:25 +0200 |
haftmann |
Haskell == is infix, not infixl
|
file |
diff |
annotate
|
Tue, 07 Sep 2010 10:05:19 +0200 |
nipkow |
expand_fun_eq -> ext_iff
|
file |
diff |
annotate
|
Thu, 02 Sep 2010 10:18:15 +0200 |
hoelzl |
Add filter_remove1
|
file |
diff |
annotate
|
Fri, 27 Aug 2010 19:34:23 +0200 |
haftmann |
renamed class/constant eq to equal; tuned some instantiations
|
file |
diff |
annotate
|