| Fri, 22 Apr 2011 15:05:04 +0200 | 
wenzelm | 
misc tuning and simplification;
 | 
file |
diff |
annotate
 | 
| Fri, 22 Apr 2011 14:30:32 +0200 | 
wenzelm | 
proper context for Quantifier1 simprocs (avoid bad ProofContext.init_global from abc655166d61);
 | 
file |
diff |
annotate
 | 
| Fri, 22 Apr 2011 13:58:13 +0200 | 
wenzelm | 
modernized Quantifier1 simproc setup;
 | 
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, 30 Mar 2011 11:32:52 +0200 | 
bulwahn | 
renewing specifications in HOL: replacing types by type_synonym
 | 
file |
diff |
annotate
 | 
| Fri, 10 Dec 2010 16:10:50 +0100 | 
haftmann | 
moved most fundamental lemmas upwards
 | 
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 13:34:51 +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
 | 
| Thu, 02 Dec 2010 14:34:58 +0100 | 
hoelzl | 
Move SUP_commute, SUP_less_iff to HOL image;
 | 
file |
diff |
annotate
 | 
| Tue, 23 Nov 2010 14:14:17 +0100 | 
hoelzl | 
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 | 
file |
diff |
annotate
 | 
| Fri, 01 Oct 2010 16:05:25 +0200 | 
haftmann | 
constant `contents` renamed to `the_elem`
 | 
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
 | 
| Wed, 08 Sep 2010 10:45:55 +0200 | 
nipkow | 
put expand_(fun/set)_eq back in as synonyms, for compatibility
 | 
file |
diff |
annotate
 | 
| Tue, 07 Sep 2010 10:05:19 +0200 | 
nipkow | 
expand_fun_eq -> ext_iff
 | 
file |
diff |
annotate
 | 
| Sat, 28 Aug 2010 16:14:32 +0200 | 
haftmann | 
formerly unnamed infix equality now named HOL.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
 | 
| Mon, 23 Aug 2010 12:13:58 +0200 | 
blanchet | 
"no_atp" fact that leads to unsound proofs
 | 
file |
diff |
annotate
 | 
| Mon, 23 Aug 2010 11:56:30 +0200 | 
blanchet | 
"no_atp" a few facts that often lead to unsound proofs
 | 
file |
diff |
annotate
 | 
| Mon, 12 Jul 2010 10:48:37 +0200 | 
haftmann | 
dropped superfluous [code del]s
 | 
file |
diff |
annotate
 | 
| Thu, 01 Jul 2010 16:54:42 +0200 | 
haftmann | 
qualified constants Set.member and Set.Collect
 | 
file |
diff |
annotate
 | 
| Tue, 08 Jun 2010 16:37:19 +0200 | 
haftmann | 
qualified types "+" and nat; qualified constants Ball, Bex, Suc, curry; modernized some specifications
 | 
file |
diff |
annotate
 | 
| Sun, 28 Mar 2010 12:50:38 -0700 | 
huffman | 
use lattice theorems to prove set theorems
 | 
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 15:44:06 +0100 | 
hoelzl | 
Added vimage_inter_cong
 | 
file |
diff |
annotate
 | 
| Mon, 01 Mar 2010 13:40:23 +0100 | 
haftmann | 
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
 | 
file |
diff |
annotate
 | 
| Thu, 11 Feb 2010 23:00:22 +0100 | 
wenzelm | 
modernized translations;
 | 
file |
diff |
annotate
 | 
| Thu, 04 Feb 2010 14:45:08 +0100 | 
hoelzl | 
Changed 'bounded unique existential quantifiers' from a constant to syntax translation.
 | 
file |
diff |
annotate
 | 
| Thu, 28 Jan 2010 11:48:49 +0100 | 
haftmann | 
new theory Algebras.thy for generic algebraic structures
 | 
file |
diff |
annotate
 | 
| Wed, 30 Dec 2009 10:24:53 +0100 | 
krauss | 
killed a few warnings
 | 
file |
diff |
annotate
 | 
| Fri, 27 Nov 2009 16:26:23 +0100 | 
berghofe | 
Removed eq_to_mono2, added not_mono.
 | 
file |
diff |
annotate
 | 
| Mon, 09 Nov 2009 15:50:15 +0000 | 
paulson | 
New theory Probability/Borel.thy, and some associated lemmas
 | 
file |
diff |
annotate
 | 
| Wed, 21 Oct 2009 11:19:11 +0100 | 
paulson | 
merged
 | 
file |
diff |
annotate
 | 
| Tue, 20 Oct 2009 16:32:51 +0100 | 
paulson | 
Some new lemmas concerning sets
 | 
file |
diff |
annotate
 | 
| Wed, 21 Oct 2009 08:16:25 +0200 | 
haftmann | 
merged
 | 
file |
diff |
annotate
 | 
| Wed, 21 Oct 2009 08:14:38 +0200 | 
haftmann | 
dropped redundant gen_ prefix
 | 
file |
diff |
annotate
 | 
| Tue, 20 Oct 2009 16:13:01 +0200 | 
haftmann | 
replaced old_style infixes eq_set, subset, union, inter and variants by generic versions
 | 
file |
diff |
annotate
 | 
| Tue, 20 Oct 2009 15:02:48 +0100 | 
paulson | 
Removal of the unused atpset concept, the atp attribute and some related code.
 | 
file |
diff |
annotate
 | 
| Wed, 07 Oct 2009 14:01:26 +0200 | 
haftmann | 
tuned proofs
 | 
file |
diff |
annotate
 | 
| Sat, 19 Sep 2009 07:38:03 +0200 | 
haftmann | 
inter and union are mere abbreviations for inf and sup
 | 
file |
diff |
annotate
 | 
| Mon, 31 Aug 2009 14:09:42 +0200 | 
nipkow | 
tuned the simp rules for Int involving insert and intervals.
 | 
file |
diff |
annotate
 | 
| Tue, 28 Jul 2009 13:37:09 +0200 | 
haftmann | 
Set.UNIV and Set.empty are mere abbreviations for top and bot
 | 
file |
diff |
annotate
 | 
| Wed, 22 Jul 2009 18:02:10 +0200 | 
haftmann | 
moved complete_lattice &c. into separate theory
 | 
file |
diff |
annotate
 | 
| Wed, 22 Jul 2009 14:20:32 +0200 | 
haftmann | 
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 | 
file |
diff |
annotate
 | 
| Tue, 21 Jul 2009 14:38:07 +0200 | 
haftmann | 
attempt for more concise setup of non-etacontracting binders
 | 
file |
diff |
annotate
 | 
| Tue, 21 Jul 2009 11:09:50 +0200 | 
haftmann | 
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 | 
file |
diff |
annotate
 | 
| Tue, 21 Jul 2009 07:54:44 +0200 | 
haftmann | 
swapped bootstrap order of UNION/Union and INTER/Inter in theory Set
 | 
file |
diff |
annotate
 | 
| Mon, 20 Jul 2009 15:24:15 +0200 | 
haftmann | 
less digestible
 | 
file |
diff |
annotate
 | 
| Mon, 20 Jul 2009 11:47:17 +0200 | 
haftmann | 
refined outline structure
 | 
file |
diff |
annotate
 | 
| Mon, 20 Jul 2009 09:52:09 +0200 | 
haftmann | 
merged
 | 
file |
diff |
annotate
 | 
| Mon, 20 Jul 2009 08:31:12 +0200 | 
haftmann | 
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 | 
file |
diff |
annotate
 | 
| Mon, 20 Jul 2009 08:32:07 +0200 | 
haftmann | 
merged
 | 
file |
diff |
annotate
 | 
| Tue, 14 Jul 2009 15:54:19 +0200 | 
haftmann | 
refinement of lattice classes
 | 
file |
diff |
annotate
 | 
| Wed, 15 Jul 2009 23:48:21 +0200 | 
wenzelm | 
more antiquotations;
 | 
file |
diff |
annotate
 | 
| Sat, 11 Jul 2009 21:33:01 +0200 | 
haftmann | 
added boolean_algebra type class; tuned lattice duals
 | 
file |
diff |
annotate
 | 
| Mon, 06 Jul 2009 21:24:30 +0200 | 
wenzelm | 
structure Thm: less pervasive names;
 | 
file |
diff |
annotate
 | 
| Mon, 15 Jun 2009 16:13:19 +0200 | 
haftmann | 
authentic syntax for Pow and image
 | 
file |
diff |
annotate
 | 
| Fri, 05 Jun 2009 08:06:03 +0200 | 
haftmann | 
merged
 | 
file |
diff |
annotate
 |