src/HOL/String.thy
Mon, 26 Feb 2018 11:52:52 +0000 haftmann dedicated append function for string literals
Wed, 10 Jan 2018 15:25:09 +0100 nipkow ran isabelle update_op on all sources
Sun, 26 Nov 2017 21:08:32 +0100 wenzelm more symbols;
Thu, 03 Aug 2017 12:50:03 +0200 haftmann lifting setup for char
Sun, 02 Jul 2017 20:13:38 +0200 haftmann proper concept of code declaration wrt. atomicity and Isar declarations
Sat, 24 Jun 2017 09:17:35 +0200 haftmann more direct construction of integer_of_num;
Mon, 06 Feb 2017 20:56:38 +0100 haftmann computation preprocessing rules to allow literals as input for computations
Tue, 20 Dec 2016 15:39:13 +0100 haftmann emphasize dedicated rewrite rules for congruences
Mon, 26 Sep 2016 07:56:54 +0200 haftmann syntactic type class for operation mod named after mod;
Sat, 19 Mar 2016 16:53:09 +0100 haftmann unified CHAR with CHR syntax
Sat, 12 Mar 2016 22:04:52 +0100 haftmann model characters directly as range 0..255
Thu, 10 Mar 2016 12:33:01 +0100 haftmann moved
Thu, 18 Feb 2016 17:52:52 +0100 haftmann more direct bootstrap of char type, still retaining the nibble representation for syntax
Mon, 07 Dec 2015 10:38:04 +0100 wenzelm isabelle update_cartouches -c -t;
Wed, 07 Oct 2015 10:02:43 +0200 blanchet disable generation of 'case_transfer' for 'nibble', due to quadratic proof -- to make 'HOL-Proofs' happier
Tue, 01 Sep 2015 22:32:58 +0200 wenzelm eliminated \<Colon>;
Thu, 27 Aug 2015 21:19:48 +0200 haftmann standardized some occurences of ancient "split" alias
Mon, 27 Jul 2015 17:44:55 +0200 wenzelm tuned signature;
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Fri, 06 Mar 2015 23:44:51 +0100 wenzelm clarified context;
Fri, 06 Mar 2015 15:58:56 +0100 wenzelm Thm.cterm_of and Thm.ctyp_of operate on local context;
Thu, 05 Feb 2015 19:44:14 +0100 haftmann slightly more standard code setup for String.literal, with explicit special case in predicate compiler
Thu, 05 Feb 2015 19:44:13 +0100 haftmann explicit type annotation avoids problems with Haskell type inference
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Wed, 29 Oct 2014 15:07:53 +0100 wenzelm modernized setup;
Thu, 11 Sep 2014 19:32:36 +0200 blanchet updated news
Wed, 03 Sep 2014 00:06:24 +0200 blanchet use 'datatype_new' in 'Main'
Fri, 04 Jul 2014 20:18:47 +0200 haftmann reduced name variants for assoc and commute on plus and mult
Mon, 30 Jun 2014 08:00:36 +0200 haftmann qualified String.explode and String.implode
Thu, 12 Jun 2014 18:47:16 +0200 nipkow added [simp]
Sun, 04 May 2014 18:14:58 +0200 blanchet renamed 'xxx_size' to 'size_xxx' for old datatype package
Fri, 07 Mar 2014 14:21:15 +0100 blanchet use balanced tuples in 'primcorec'
Fri, 21 Feb 2014 00:09:56 +0100 blanchet adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'
Wed, 12 Feb 2014 10:59:25 +0100 Andreas Lochbihler merged
Wed, 12 Feb 2014 08:56:38 +0100 Andreas Lochbihler make lifting setup for String.literal local to prevent transfer from replacing STR ''...'' literals
Wed, 12 Feb 2014 08:35:57 +0100 blanchet adapted theories to 'xxx_case' to 'case_xxx'
Wed, 15 Jan 2014 23:25:28 +0100 wenzelm added \<newline> symbol, which is used for char/string literals in HOL;
Wed, 20 Nov 2013 11:10:05 +0100 Andreas Lochbihler setup lifting/transfer for String.literal
Wed, 09 Oct 2013 15:33:20 +0200 Andreas Lochbihler add congruence rule to prevent code_simp from looping
Thu, 08 Aug 2013 16:10:05 +0200 Andreas Lochbihler abort execution of generated code with explicit exception message
Sun, 23 Jun 2013 21:16:07 +0200 haftmann migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
Tue, 11 Jun 2013 21:07:53 +0200 haftmann reflexive nbe equation for equality on String.literal
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Fri, 15 Feb 2013 11:47:33 +0100 haftmann systematic conversions between nat and nibble/char;
Mon, 22 Oct 2012 22:24:34 +0200 haftmann incorporated constant chars into instantiation proof for enum;
Sat, 20 Oct 2012 09:12:16 +0200 haftmann moved quite generic material from theory Enum to more appropriate places
Fri, 12 Oct 2012 18:58:20 +0200 wenzelm discontinued obsolete typedef (open) syntax;
Wed, 22 Aug 2012 22:55:41 +0200 wenzelm prefer ML_file over old uses;
Wed, 15 Feb 2012 13:24:22 +0100 wenzelm renamed "xstr" to "str_token";
Mon, 14 Nov 2011 17:48:26 +0100 wenzelm inner syntax positions for string literals;
Wed, 19 Oct 2011 08:37:29 +0200 bulwahn removing old code generator setup for strings
Thu, 18 Aug 2011 13:55:26 +0200 haftmann observe distinction between sets and predicates more properly
Thu, 21 Apr 2011 12:56:27 +0200 wenzelm discontinuend obsolete Thm.definitionK, which was hardly ever well-defined;
Tue, 19 Apr 2011 23:57:28 +0200 wenzelm eliminated Codegen.mode in favour of explicit argument;
Wed, 30 Mar 2011 11:32:52 +0200 bulwahn renewing specifications in HOL: replacing types by type_synonym
Thu, 10 Feb 2011 10:32:12 +0100 haftmann reverted cs. 0a3fa8fbcdc5 -- motivation is unreconstructable, produces confusion in user space
Mon, 20 Sep 2010 16:05:25 +0200 wenzelm renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
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
Fri, 10 Sep 2010 10:59:09 +0200 bulwahn fiddling with the correct setup for String.literal
Fri, 10 Sep 2010 10:21:25 +0200 haftmann Haskell == is infix, not infixl
less more (0) -60 tip