src/HOL/Fun.thy
Thu, 07 Jul 2011 21:53:53 +0200 added translation to fix critical pair between abbreviations for surj and ~=
Fri, 20 May 2011 21:38:32 +0200 add surj_vimage_empty
Tue, 05 Apr 2011 11:44:34 +0200 added "no_atp" to Cantor's paradox
Fri, 21 Jan 2011 09:44:12 +0100 moved theorem
Tue, 11 Jan 2011 14:12:37 +0100 "enriched_type" replaces less specific "type_lifting"
Fri, 17 Dec 2010 17:43:54 +0100 replaced command 'nonterminals' by slightly modernized version 'nonterminal';
Mon, 06 Dec 2010 09:25:05 +0100 moved bootstrap of type_lifting to Fun
Mon, 06 Dec 2010 09:19:10 +0100 replace `type_mapper` by the more adequate `type_lifting`
Fri, 26 Nov 2010 21:09:36 +0100 keep private things private, without comments;
Tue, 23 Nov 2010 14:14:17 +0100 Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
Mon, 22 Nov 2010 10:34:33 +0100 Replace surj by abbreviation; remove surj_on.
Thu, 18 Nov 2010 17:01:15 +0100 map_fun combinator in theory Fun
Mon, 13 Sep 2010 11:13:15 +0200 renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
Wed, 08 Sep 2010 10:45:55 +0200 put expand_(fun/set)_eq back in as synonyms, for compatibility
Tue, 07 Sep 2010 10:05:19 +0200 expand_fun_eq -> ext_iff
Thu, 02 Sep 2010 21:08:31 +0200 Revert bij_betw changes to simp set (Problem in afp/Ordinals_and_Cardinals)
Thu, 02 Sep 2010 11:54:09 +0200 Introduce surj_on and replace surj and bij by abbreviations.
Thu, 02 Sep 2010 10:45:51 +0200 Permutation implies bij function
Thu, 02 Sep 2010 10:36:45 +0200 bij <--> bij_betw
Fri, 20 Aug 2010 17:46:55 +0200 inj_comp and inj_fun
Mon, 12 Jul 2010 10:48:37 +0200 dropped superfluous [code del]s
Fri, 09 Jul 2010 08:11:10 +0200 nicer xsymbol syntax for fcomp and scomp
Fri, 16 Apr 2010 21:28:09 +0200 replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
Fri, 05 Mar 2010 17:49:10 +0100 generalized inj_uminus; added strict_mono_imp_inj_on
Thu, 04 Mar 2010 19:43:51 +0100 Rewrite rules for images of minus of intervals
Mon, 01 Mar 2010 13:40:23 +0100 replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
Thu, 11 Feb 2010 23:00:22 +0100 modernized translations;
Wed, 30 Dec 2009 10:24:53 +0100 killed a few warnings
Mon, 21 Dec 2009 08:32:22 +0100 merged
Mon, 21 Dec 2009 08:32:03 +0100 moved lemmas o_eq_dest, o_eq_elim here
Fri, 18 Dec 2009 18:48:27 -0800 add lemma swap_triple
Wed, 16 Dec 2009 14:38:35 -0800 declare swap_self [simp], add lemma comp_swap
Thu, 29 Oct 2009 11:41:36 +0100 moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
Thu, 22 Oct 2009 09:27:48 +0200 inv_onto -> inv_into
Tue, 20 Oct 2009 16:32:51 +0100 Some new lemmas concerning sets
Mon, 19 Oct 2009 16:43:45 +0200 Renamed inv to the_inv and turned it into an abbreviation (based on the_inv_onto).
Sun, 18 Oct 2009 12:07:25 +0200 Inv -> inv_onto, inv abbr. inv_onto UNIV.
Sat, 17 Oct 2009 13:46:39 +0200 added the_inv_onto
Tue, 29 Sep 2009 16:24:36 +0200 explicit indication of Unsynchronized.ref;
Thu, 10 Sep 2009 15:23:07 +0200 early bootstrap of generic transfer procedure
Mon, 10 Aug 2009 17:00:41 +0200 new lemma bij_comp
Wed, 22 Jul 2009 18:02:10 +0200 moved complete_lattice &c. into separate theory
Mon, 06 Jul 2009 14:19:13 +0200 moved Inductive.myinv to Fun.inv; tuned
Tue, 23 Jun 2009 12:09:30 +0200 uniformly capitialized names for subdirectories
Wed, 10 Jun 2009 15:04:33 +0200 separate directory for datatype package
Thu, 04 Jun 2009 13:26:32 +0200 A few finite lemmas
Tue, 19 May 2009 13:57:31 +0200 pretty printing of functional combinators for evaluation code
Sat, 09 May 2009 07:25:22 +0200 lemmas by Andreas Lochbihler
Thu, 05 Mar 2009 08:23:08 +0100 dropped Id
Fri, 31 Oct 2008 10:35:30 +0100 Replaced arbitrary by undefined.
Fri, 10 Oct 2008 06:45:53 +0200 `code func` now just `code`
Mon, 23 Jun 2008 23:45:39 +0200 Logic.all/mk_equals/mk_implies;
Fri, 13 Jun 2008 15:22:07 +0200 hide -> hide (open)
Thu, 12 Jun 2008 14:10:41 +0200 Hid swap
Tue, 10 Jun 2008 19:15:18 +0200 tuned proofs -- case_tac *is* available here;
Tue, 10 Jun 2008 15:30:56 +0200 removed some dubious code lemmas
Wed, 09 Apr 2008 08:10:11 +0200 removed syntax from monad combinators; renamed mbind to scomp
Thu, 20 Mar 2008 12:04:53 +0100 added forward composition
Wed, 19 Mar 2008 22:50:42 +0100 more antiquotations;
Tue, 26 Feb 2008 20:38:12 +0100 moved some set lemmas to Set.thy