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
|
Wed, 25 Aug 2010 18:36:22 +0200 |
wenzelm |
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
|
file |
diff |
annotate
|
Mon, 19 Jul 2010 11:55:43 +0200 |
haftmann |
Scala: subtle difference in printing strings vs. complex mixfix syntax
|
file |
diff |
annotate
|
Mon, 12 Jul 2010 10:48:37 +0200 |
haftmann |
dropped superfluous [code del]s
|
file |
diff |
annotate
|
Mon, 28 Jun 2010 15:32:26 +0200 |
haftmann |
put section on distinctness before listsum; refined code generation operations; dropped ancient infix mem
|
file |
diff |
annotate
|
Fri, 18 Jun 2010 21:22:05 +0200 |
haftmann |
merged
|
file |
diff |
annotate
|
Fri, 18 Jun 2010 09:21:41 +0200 |
haftmann |
made List.thy a join point in the theory graph
|
file |
diff |
annotate
|
Fri, 18 Jun 2010 20:22:06 +0200 |
nipkow |
tuned set_replicate lemmas
|
file |
diff |
annotate
|
Fri, 18 Jun 2010 14:14:42 +0200 |
nipkow |
merged
|
file |
diff |
annotate
|
Fri, 18 Jun 2010 14:14:29 +0200 |
nipkow |
added lemmas
|
file |
diff |
annotate
|
Thu, 17 Jun 2010 16:15:15 +0200 |
haftmann |
rev is reverse in Haskell
|
file |
diff |
annotate
|
Mon, 14 Jun 2010 12:01:30 +0200 |
haftmann |
use various predefined Haskell operations when generating code
|
file |
diff |
annotate
|
Sat, 12 Jun 2010 15:47:50 +0200 |
haftmann |
declare lexn.simps [code del]
|
file |
diff |
annotate
|
Wed, 02 Jun 2010 15:35:14 +0200 |
haftmann |
induction over non-empty lists
|
file |
diff |
annotate
|
Wed, 26 May 2010 11:59:06 +0200 |
haftmann |
more convenient order of code equations
|
file |
diff |
annotate
|
Mon, 24 May 2010 13:48:57 +0200 |
haftmann |
more lemmas
|
file |
diff |
annotate
|
Thu, 20 May 2010 16:35:52 +0200 |
haftmann |
turned old-style mem into an input abbreviation
|
file |
diff |
annotate
|
Fri, 14 May 2010 22:46:41 +0200 |
nipkow |
added listsum lemmas
|
file |
diff |
annotate
|
Thu, 13 May 2010 14:34:05 +0200 |
nipkow |
Multiset: renamed, added and tuned lemmas;
|
file |
diff |
annotate
|
Wed, 12 May 2010 11:17:59 +0200 |
haftmann |
added lemmas concerning last, butlast, insort
|
file |
diff |
annotate
|
Tue, 20 Apr 2010 17:58:34 +0200 |
hoelzl |
Generalize swap_inj_on; add simps for Times; add Ex_list_of_length, log_inj; Added missing locale edges for linordered semiring with 1.
|
file |
diff |
annotate
|
Thu, 22 Apr 2010 09:30:39 +0200 |
haftmann |
lemmas concerning remdups
|
file |
diff |
annotate
|
Mon, 19 Apr 2010 07:38:35 +0200 |
haftmann |
merged
|
file |
diff |
annotate
|
Mon, 19 Apr 2010 07:38:08 +0200 |
haftmann |
more convenient equations for zip
|
file |
diff |
annotate
|
Fri, 16 Apr 2010 21:28:09 +0200 |
wenzelm |
replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
|
file |
diff |
annotate
|
Thu, 15 Apr 2010 16:55:12 +0200 |
Cezary Kaliszyk |
Respectfullness and preservation of list_rel
|
file |
diff |
annotate
|
Thu, 18 Mar 2010 12:58:52 +0100 |
blanchet |
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
|
file |
diff |
annotate
|
Wed, 17 Mar 2010 19:37:44 +0100 |
blanchet |
renamed "ATP_Linkup" theory to "Sledgehammer"
|
file |
diff |
annotate
|
Sat, 06 Mar 2010 09:58:33 +0100 |
haftmann |
added insort_insert
|
file |
diff |
annotate
|
Fri, 05 Mar 2010 17:55:14 +0100 |
haftmann |
moved lemma map_sorted_distinct_set_unique
|
file |
diff |
annotate
|
Tue, 02 Mar 2010 17:36:16 +0000 |
paulson |
Slightly generalised a theorem
|
file |
diff |
annotate
|
Mon, 22 Feb 2010 09:24:20 +0100 |
haftmann |
merged
|
file |
diff |
annotate
|
Sat, 20 Feb 2010 21:13:29 +0100 |
haftmann |
lemma distinct_insert
|
file |
diff |
annotate
|
Mon, 22 Feb 2010 09:17:49 +0100 |
haftmann |
merged
|
file |
diff |
annotate
|
Fri, 19 Feb 2010 14:47:01 +0100 |
haftmann |
moved remaning class operations from Algebras.thy to Groups.thy
|
file |
diff |
annotate
|
Sun, 21 Feb 2010 21:10:01 +0100 |
wenzelm |
adapted to authentic syntax;
|
file |
diff |
annotate
|