| Fri, 04 Jan 2019 23:22:53 +0100 | 
wenzelm | 
isabelle update -u control_cartouches;
 | 
file |
diff |
annotate
 | 
| Tue, 24 Apr 2018 14:17:58 +0000 | 
haftmann | 
proper datatype for 8-bit characters
 | 
file |
diff |
annotate
 | 
| Wed, 10 Jan 2018 15:25:09 +0100 | 
nipkow | 
ran isabelle update_op on all sources
 | 
file |
diff |
annotate
 | 
| Sun, 26 Nov 2017 21:08:32 +0100 | 
wenzelm | 
more symbols;
 | 
file |
diff |
annotate
 | 
| Mon, 26 Sep 2016 07:56:54 +0200 | 
haftmann | 
syntactic type class for operation mod named after mod;
 | 
file |
diff |
annotate
 | 
| Thu, 01 Sep 2016 21:28:55 +0200 | 
wenzelm | 
tuned headers;
 | 
file |
diff |
annotate
 | 
| Sat, 12 Mar 2016 22:04:52 +0100 | 
haftmann | 
model characters directly as range 0..255
 | 
file |
diff |
annotate
 | 
| Thu, 05 Nov 2015 10:39:49 +0100 | 
wenzelm | 
isabelle update_cartouches -c -t;
 | 
file |
diff |
annotate
 | 
| Tue, 13 Oct 2015 09:21:15 +0200 | 
haftmann | 
prod_case as canonical name for product type eliminator
 | 
file |
diff |
annotate
 | 
| Tue, 15 Sep 2015 22:25:06 +0200 | 
Andreas Lochbihler | 
avoid module dependency cycles
 | 
file |
diff |
annotate
 | 
| Wed, 09 Sep 2015 17:07:44 +0200 | 
Andreas Lochbihler | 
reactivate examples with predicate compiler and quickcheck
 | 
file |
diff |
annotate
 | 
| Sun, 06 Sep 2015 22:14:51 +0200 | 
haftmann | 
prefer "uncurry" as canonical name for case distinction on products in combinatorial view
 | 
file |
diff |
annotate
 | 
| Wed, 17 Jun 2015 11:03:05 +0200 | 
wenzelm | 
isabelle update_cartouches;
 | 
file |
diff |
annotate
 | 
| Mon, 01 Jun 2015 18:59:21 +0200 | 
haftmann | 
separate class for division operator, with particular syntax added in more specific classes
 | 
file |
diff |
annotate
 | 
| Mon, 13 Apr 2015 12:15:29 +0200 | 
hoelzl | 
predicate compiler: ignore Abs_filter and Rep_filter
 | 
file |
diff |
annotate
 | 
| Thu, 24 Apr 2014 00:23:38 +0200 | 
blanchet | 
avoid name shadowing
 | 
file |
diff |
annotate
 | 
| Thu, 13 Mar 2014 07:07:07 +0100 | 
nipkow | 
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 | 
file |
diff |
annotate
 | 
| Wed, 12 Feb 2014 08:35:57 +0100 | 
blanchet | 
renamed '{prod,sum,bool,unit}_case' to 'case_...'
 | 
file |
diff |
annotate
 | 
| Tue, 19 Nov 2013 10:05:53 +0100 | 
haftmann | 
eliminiated neg_numeral in favour of - (numeral _)
 | 
file |
diff |
annotate
 | 
| Fri, 15 Feb 2013 08:31:31 +0100 | 
haftmann | 
two target language numeral types: integer and natural, as replacement for code_numeral;
 | 
file |
diff |
annotate
 | 
| Wed, 01 Aug 2012 22:12:29 +0200 | 
wenzelm | 
fixed document;
 | 
file |
diff |
annotate
 | 
| Mon, 30 Apr 2012 12:14:51 +0200 | 
bulwahn | 
removing obsolete setup for sets now that sets are executable
 | 
file |
diff |
annotate
 | 
| Sun, 25 Mar 2012 20:15:39 +0200 | 
huffman | 
merged fork with new numeral representation (see NEWS)
 | 
file |
diff |
annotate
 | 
| Tue, 13 Mar 2012 16:56:56 +0100 | 
wenzelm | 
prefer abs_def over def_raw;
 | 
file |
diff |
annotate
 | 
| Mon, 12 Mar 2012 21:41:11 +0100 | 
noschinl | 
tuned proofs
 | 
file |
diff |
annotate
 | 
| Sat, 24 Dec 2011 15:53:10 +0100 | 
haftmann | 
adjusted to set/pred distinction by means of type constructor `set`
 | 
file |
diff |
annotate
 | 
| Fri, 11 Nov 2011 12:10:49 +0100 | 
bulwahn | 
using more conventional names for monad plus operations
 | 
file |
diff |
annotate
 | 
| Fri, 21 Oct 2011 11:17:14 +0200 | 
bulwahn | 
replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed
 | 
file |
diff |
annotate
 | 
| Wed, 14 Sep 2011 10:08:52 -0400 | 
hoelzl | 
renamed Complete_Lattices lemmas, removed legacy names
 | 
file |
diff |
annotate
 | 
| Mon, 12 Sep 2011 07:55:43 +0200 | 
nipkow | 
new fastforce replacing fastsimp - less confusing name
 | 
file |
diff |
annotate
 | 
| Wed, 17 Aug 2011 18:05:31 +0200 | 
wenzelm | 
modernized signature of Term.absfree/absdummy;
 | 
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
 | 
| Mon, 15 Nov 2010 13:40:12 +0100 | 
bulwahn | 
ignoring the constant STR in the predicate compiler
 | 
file |
diff |
annotate
 | 
| Thu, 21 Oct 2010 19:13:11 +0200 | 
bulwahn | 
adapting alternative_defs, predicate_compile_quickcheck, examples and code_prolog
 | 
file |
diff |
annotate
 | 
| Thu, 23 Sep 2010 14:50:14 +0200 | 
bulwahn | 
handling equivalences smarter in the predicate compiler
 | 
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
 | 
| Tue, 07 Sep 2010 10:05:19 +0200 | 
nipkow | 
expand_fun_eq -> ext_iff
 | 
file |
diff |
annotate
 | 
| Mon, 28 Jun 2010 15:03:07 +0200 | 
haftmann | 
merged constants "split" and "prod_case"
 | 
file |
diff |
annotate
 | 
| Wed, 21 Apr 2010 12:10:52 +0200 | 
bulwahn | 
added further inlining of boolean constants to the predicate compiler
 | 
file |
diff |
annotate
 | 
| Wed, 21 Apr 2010 12:10:52 +0200 | 
bulwahn | 
added peephole optimisations to the predicate compiler; added structure Predicate_Compile_Simps for peephole optimisations
 | 
file |
diff |
annotate
 | 
| Wed, 31 Mar 2010 16:44:41 +0200 | 
bulwahn | 
adding setup for handling arithmetic of natural numbers and integers precisely and more efficiently in the predicate compiler; changed alternative size_list definition for predicate compiler
 | 
file |
diff |
annotate
 | 
| Wed, 24 Mar 2010 17:40:43 +0100 | 
bulwahn | 
moved further predicate compile files to HOL-Library
 | 
file |
diff |
annotate
 |