Wed, 26 Apr 2017 15:53:35 +0100 |
paulson |
Further new material. The simprule status of some exp and ln identities was reverted.
|
file |
diff |
annotate
|
Sun, 05 Mar 2017 10:57:51 +0100 |
nipkow |
added numeral_powr_numeral
|
file |
diff |
annotate
|
Sun, 16 Oct 2016 09:31:06 +0200 |
haftmann |
eliminated irregular aliasses
|
file |
diff |
annotate
|
Sun, 16 Oct 2016 09:31:04 +0200 |
haftmann |
more standardized names
|
file |
diff |
annotate
|
Fri, 12 Aug 2016 09:57:09 +0200 |
nipkow |
tuned
|
file |
diff |
annotate
|
Fri, 12 Aug 2016 08:20:17 +0200 |
nipkow |
Extracted floorlog and bitlen to separate theory Log_Nat
|
file |
diff |
annotate
|
Fri, 05 Aug 2016 12:27:51 +0200 |
nipkow |
fixed floor proofs
|
file |
diff |
annotate
|
Fri, 05 Aug 2016 09:05:03 +0200 |
nipkow |
more lemmas
|
file |
diff |
annotate
|
Fri, 24 Jun 2016 20:27:57 +0200 |
wenzelm |
misc tuning and modernization;
|
file |
diff |
annotate
|
Wed, 08 Jun 2016 16:46:48 +0200 |
immler |
generalized bitlen to floor of log
|
file |
diff |
annotate
|
Mon, 25 Apr 2016 16:09:26 +0200 |
wenzelm |
eliminated old 'def';
|
file |
diff |
annotate
|
Fri, 26 Feb 2016 11:53:45 +0100 |
immler |
finite precision computation to determine sign for comparison
|
file |
diff |
annotate
|
Fri, 26 Feb 2016 11:53:45 +0100 |
immler |
positive precision for truncate; fixed precision for approximation of rationals; code for truncate
|
file |
diff |
annotate
|
Fri, 26 Feb 2016 11:53:42 +0100 |
immler |
compute_real_of_float has not been used as code equation
|
file |
diff |
annotate
|
Tue, 23 Feb 2016 16:25:08 +0100 |
nipkow |
more canonical names
|
file |
diff |
annotate
|
Wed, 17 Feb 2016 21:51:57 +0100 |
haftmann |
dropped various legacy fact bindings
|
file |
diff |
annotate
|
Mon, 28 Dec 2015 01:28:28 +0100 |
wenzelm |
more symbols;
|
file |
diff |
annotate
|
Sun, 27 Dec 2015 21:46:36 +0100 |
wenzelm |
prefer symbols for "floor", "ceiling";
|
file |
diff |
annotate
|
Mon, 07 Dec 2015 10:38:04 +0100 |
wenzelm |
isabelle update_cartouches -c -t;
|
file |
diff |
annotate
|
Tue, 01 Dec 2015 14:09:10 +0000 |
paulson |
Removal of redundant lemmas (diff_less_iff, diff_le_iff) and of the abbreviation Exp. Addition of some new material.
|
file |
diff |
annotate
|
Fri, 13 Nov 2015 12:27:13 +0000 |
paulson |
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
|
file |
diff |
annotate
|
Wed, 11 Nov 2015 17:11:50 +0000 |
paulson |
new conversion theorems for int, nat to float
|
file |
diff |
annotate
|
Tue, 10 Nov 2015 14:18:41 +0000 |
paulson |
Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
|
file |
diff |
annotate
|
Sat, 08 Aug 2015 10:51:33 +0200 |
haftmann |
direct bootstrap of integer division from natural division
|
file |
diff |
annotate
|
Thu, 09 Jul 2015 00:40:57 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Mon, 06 Jul 2015 22:57:34 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Wed, 17 Jun 2015 11:03:05 +0200 |
wenzelm |
isabelle update_cartouches;
|
file |
diff |
annotate
|
Sun, 07 Jun 2015 14:36:36 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Sat, 11 Apr 2015 11:56:40 +0100 |
paulson |
Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
|
file |
diff |
annotate
|
Thu, 09 Apr 2015 09:12:47 +0200 |
haftmann |
conversion between division on nat/int and division in archmedean fields
|
file |
diff |
annotate
|
Wed, 18 Feb 2015 22:46:47 +0100 |
haftmann |
inlined rules to free user-space from technical names
|
file |
diff |
annotate
|
Fri, 06 Feb 2015 17:57:03 +0100 |
haftmann |
default abstypes and default abstract equations make technical (no_code) annotation superfluous
|
file |
diff |
annotate
|
Wed, 12 Nov 2014 17:37:43 +0100 |
immler |
tuned proofs
|
file |
diff |
annotate
|
Wed, 12 Nov 2014 17:37:43 +0100 |
immler |
quickcheck setup for float, inspired by rat::{exhaustive,full_exhaustive,random}
|
file |
diff |
annotate
|
Wed, 12 Nov 2014 17:37:43 +0100 |
immler |
truncate intermediate results in horner to improve performance of approximate;
|
file |
diff |
annotate
|
Wed, 12 Nov 2014 17:36:29 +0100 |
immler |
simplified computations based on round_up by reducing to round_down;
|
file |
diff |
annotate
|
Sun, 02 Nov 2014 17:20:45 +0100 |
wenzelm |
modernized header;
|
file |
diff |
annotate
|
Thu, 30 Oct 2014 21:02:01 +0100 |
haftmann |
more simp rules concerning dvd and even/odd
|
file |
diff |
annotate
|
Sun, 21 Sep 2014 16:56:11 +0200 |
haftmann |
explicit separation of signed and unsigned numerals using existing lexical categories num and xnum
|
file |
diff |
annotate
|
Mon, 25 Aug 2014 14:24:05 +0200 |
hoelzl |
introduce real_of typeclass for real :: 'a => real
|
file |
diff |
annotate
|
Tue, 05 Aug 2014 12:56:15 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Fri, 04 Jul 2014 20:18:47 +0200 |
haftmann |
reduced name variants for assoc and commute on plus and mult
|
file |
diff |
annotate
|
Wed, 11 Jun 2014 14:24:23 +1000 |
Thomas Sewell |
Hypsubst preserves equality hypotheses
|
file |
diff |
annotate
|
Mon, 28 Apr 2014 17:50:03 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Mon, 14 Apr 2014 13:08:17 +0200 |
hoelzl |
added divide_nonneg_nonneg and co; made it a simp rule
|
file |
diff |
annotate
|
Sat, 12 Apr 2014 17:26:27 +0200 |
nipkow |
made mult_pos_pos a simp rule
|
file |
diff |
annotate
|
Fri, 11 Apr 2014 13:36:57 +0200 |
nipkow |
made mult_nonneg_nonneg a simp rule
|
file |
diff |
annotate
|
Wed, 09 Apr 2014 09:37:47 +0200 |
hoelzl |
revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
|
file |
diff |
annotate
|
Fri, 04 Apr 2014 17:58:25 +0100 |
paulson |
divide_minus_left divide_minus_right are in field_simps but are not default simprules
|
file |
diff |
annotate
|
Thu, 06 Mar 2014 15:40:33 +0100 |
blanchet |
renamed 'fun_rel' to 'rel_fun'
|
file |
diff |
annotate
|
Tue, 18 Feb 2014 23:03:50 +0100 |
kuncar |
simplify proofs because of the stronger reflexivity prover
|
file |
diff |
annotate
|
Mon, 16 Dec 2013 17:08:22 +0100 |
immler |
monotonicity of rounding and truncating float
|
file |
diff |
annotate
|
Mon, 16 Dec 2013 17:08:22 +0100 |
immler |
Float: prevent unnecessary large numbers when adding 0
|
file |
diff |
annotate
|
Mon, 16 Dec 2013 17:08:22 +0100 |
immler |
additional definitions and lemmas for Float
|
file |
diff |
annotate
|
Tue, 19 Nov 2013 10:05:53 +0100 |
haftmann |
eliminiated neg_numeral in favour of - (numeral _)
|
file |
diff |
annotate
|
Fri, 01 Nov 2013 18:51:14 +0100 |
haftmann |
more simplification rules on unary and binary minus
|
file |
diff |
annotate
|
Tue, 03 Sep 2013 22:04:23 +0200 |
wenzelm |
tuned proofs -- less guessing;
|
file |
diff |
annotate
|
Tue, 27 Aug 2013 14:37:56 +0200 |
hoelzl |
renamed typeclass dense_linorder to unbounded_dense_linorder
|
file |
diff |
annotate
|
Tue, 26 Mar 2013 20:02:02 +0100 |
wenzelm |
tuned imports;
|
file |
diff |
annotate
|
Fri, 08 Mar 2013 13:21:06 +0100 |
kuncar |
patch Isabelle ditribution to conform to changes regarding the parametricity
|
file |
diff |
annotate
|