Tue, 13 Sep 2011 17:07:33 -0700 |
huffman |
tuned proofs
|
file |
diff |
annotate
|
Mon, 08 Aug 2011 17:23:15 +0200 |
wenzelm |
misc tuning -- eliminated old-fashioned rep_thm;
|
file |
diff |
annotate
|
Wed, 03 Aug 2011 23:21:52 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
Sat, 16 Jul 2011 22:04:02 +0200 |
haftmann |
consolidated bot and top classes, tuned notation
|
file |
diff |
annotate
|
Wed, 13 Jul 2011 23:49:56 +0200 |
haftmann |
uniqueness lemmas for bot and top
|
file |
diff |
annotate
|
Wed, 13 Jul 2011 19:43:12 +0200 |
haftmann |
moved lemmas bot_less and less_top to classes bot and top respectively
|
file |
diff |
annotate
|
Wed, 13 Jul 2011 19:40:18 +0200 |
haftmann |
tightened specification of classes bot and top: uniqueness of top and bot elements
|
file |
diff |
annotate
|
Wed, 29 Jun 2011 21:34:16 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Wed, 29 Jun 2011 20:39:41 +0200 |
wenzelm |
simplified/unified Simplifier.mk_solver;
|
file |
diff |
annotate
|
Fri, 13 May 2011 23:58:40 +0200 |
wenzelm |
clarified map_simpset versus Simplifier.map_simpset_global;
|
file |
diff |
annotate
|
Fri, 08 Apr 2011 14:20:57 +0200 |
wenzelm |
discontinued special treatment of structure Mixfix;
|
file |
diff |
annotate
|
Fri, 08 Apr 2011 13:31:16 +0200 |
wenzelm |
explicit structure Syntax_Trans;
|
file |
diff |
annotate
|
Wed, 08 Dec 2010 15:05:46 +0100 |
haftmann |
bot comes before top, inf before sup etc.
|
file |
diff |
annotate
|
Wed, 08 Dec 2010 14:52:23 +0100 |
haftmann |
nice syntax for lattice INFI, SUPR;
|
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
|
Fri, 27 Aug 2010 10:56:46 +0200 |
haftmann |
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
|
file |
diff |
annotate
|
Thu, 26 Aug 2010 20:51:17 +0200 |
haftmann |
formerly unnamed infix impliciation now named HOL.implies
|
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
|
Tue, 24 Aug 2010 14:41:37 +0200 |
hoelzl |
moved generic lemmas in Probability to HOL
|
file |
diff |
annotate
|
Mon, 23 Aug 2010 14:21:57 +0200 |
blanchet |
"no_atp" fact that leads to unsound proofs in Sledgehammer
|
file |
diff |
annotate
|
Mon, 12 Jul 2010 10:48:37 +0200 |
haftmann |
dropped superfluous [code del]s
|
file |
diff |
annotate
|
Mon, 17 May 2010 23:54:15 +0200 |
wenzelm |
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
|
file |
diff |
annotate
|
Tue, 04 May 2010 08:55:43 +0200 |
haftmann |
locale predicates of classes carry a mandatory "class" prefix
|
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
|
Thu, 04 Mar 2010 18:42:39 +0100 |
hoelzl |
Add dense_le, dense_le_bounded, field_le_mult_one_interval.
|
file |
diff |
annotate
|
Thu, 25 Feb 2010 22:32:09 +0100 |
wenzelm |
more antiquotations;
|
file |
diff |
annotate
|
Mon, 22 Feb 2010 15:53:18 +0100 |
haftmann |
distributed theory Algebras to theories Groups and Lattices
|
file |
diff |
annotate
|
Thu, 11 Feb 2010 23:00:22 +0100 |
wenzelm |
modernized translations;
|
file |
diff |
annotate
|
Wed, 10 Feb 2010 14:12:04 +0100 |
haftmann |
moved less_eq, less to Orderings.thy; moved abs, sgn to Groups.thy
|
file |
diff |
annotate
|
Fri, 05 Feb 2010 14:33:50 +0100 |
haftmann |
more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
|
file |
diff |
annotate
|
Thu, 28 Jan 2010 11:48:49 +0100 |
haftmann |
new theory Algebras.thy for generic algebraic structures
|
file |
diff |
annotate
|
Mon, 04 Jan 2010 16:00:23 +0100 |
haftmann |
moved name duplicates to end of theory; reduced warning noise
|
file |
diff |
annotate
|
Fri, 11 Dec 2009 14:43:56 +0100 |
haftmann |
moved predicate rules to Predicate.thy; weakened default dest rule predicate1D (is not that reliable wrt. sets)
|
file |
diff |
annotate
|
Sun, 08 Nov 2009 16:30:41 +0100 |
wenzelm |
adapted Generic_Data, Proof_Data;
|
file |
diff |
annotate
|
Sat, 17 Oct 2009 14:43:18 +0200 |
wenzelm |
eliminated hard tabulators, guessing at each author's individual tab-width;
|
file |
diff |
annotate
|
Fri, 09 Oct 2009 13:34:34 +0200 |
haftmann |
tuned order of lemmas
|
file |
diff |
annotate
|
Wed, 07 Oct 2009 14:01:26 +0200 |
haftmann |
added bot_boolE, top_boolI
|
file |
diff |
annotate
|
Sun, 26 Jul 2009 22:28:31 +0200 |
wenzelm |
replaced old METAHYPS by FOCUS;
|
file |
diff |
annotate
|
Tue, 14 Jul 2009 10:54:04 +0200 |
haftmann |
code attributes use common underscore convention
|
file |
diff |
annotate
|
Wed, 15 Apr 2009 15:52:37 +0200 |
haftmann |
code generator bootstrap theory src/Tools/Code_Generator.thy
|
file |
diff |
annotate
|
Mon, 30 Mar 2009 22:48:15 +0200 |
wenzelm |
simplified 'print_orders' command;
|
file |
diff |
annotate
|
Thu, 26 Mar 2009 14:14:02 +0100 |
wenzelm |
simplified attribute and method setup: eliminating bottom-up styles makes it easier to keep things in one place, and also SML/NJ happy;
|
file |
diff |
annotate
|
Sun, 15 Mar 2009 15:59:44 +0100 |
wenzelm |
simplified attribute setup;
|
file |
diff |
annotate
|
Fri, 13 Mar 2009 23:50:05 +0100 |
wenzelm |
simplified method setup;
|
file |
diff |
annotate
|
Fri, 13 Mar 2009 19:58:26 +0100 |
wenzelm |
unified type Proof.method and pervasive METHOD combinators;
|
file |
diff |
annotate
|
Fri, 06 Mar 2009 14:33:19 +0100 |
haftmann |
added strict_mono predicate
|
file |
diff |
annotate
|
Thu, 26 Feb 2009 16:32:46 +0100 |
berghofe |
Fixed nonexhaustive match problem in decomp, to make it fail more gracefully
|
file |
diff |
annotate
|
Fri, 06 Feb 2009 15:15:32 +0100 |
haftmann |
session Reflecion renamed to Decision_Procs, moved Dense_Linear_Order there
|
file |
diff |
annotate
|
Wed, 21 Jan 2009 16:47:31 +0100 |
haftmann |
dropped ID
|
file |
diff |
annotate
|
Mon, 17 Nov 2008 17:00:55 +0100 |
haftmann |
tuned unfold_locales invocation
|
file |
diff |
annotate
|
Fri, 24 Oct 2008 17:48:37 +0200 |
haftmann |
new classes "top" and "bot"
|
file |
diff |
annotate
|
Fri, 10 Oct 2008 06:45:53 +0200 |
haftmann |
`code func` now just `code`
|
file |
diff |
annotate
|
Tue, 07 Oct 2008 16:07:21 +0200 |
haftmann |
tuned min/max code generation
|
file |
diff |
annotate
|
Mon, 11 Aug 2008 14:49:53 +0200 |
haftmann |
moved class wellorder to theory Orderings
|
file |
diff |
annotate
|
Tue, 29 Jul 2008 08:15:38 +0200 |
haftmann |
declare
|
file |
diff |
annotate
|
Fri, 25 Jul 2008 12:03:34 +0200 |
haftmann |
added class preorder
|
file |
diff |
annotate
|
Fri, 20 Jun 2008 21:00:21 +0200 |
haftmann |
streamlined definitions
|
file |
diff |
annotate
|
Tue, 10 Jun 2008 15:30:58 +0200 |
haftmann |
localized Least in Orderings.thy
|
file |
diff |
annotate
|
Wed, 07 May 2008 10:56:38 +0200 |
berghofe |
- Now imports Code_Setup, rather than Set and Fun, since the theorems
|
file |
diff |
annotate
|
Sat, 29 Mar 2008 22:55:49 +0100 |
wenzelm |
purely functional setup of claset/simpset/clasimpset;
|
file |
diff |
annotate
|