Mon, 09 Jan 2017 18:53:06 +0100 |
haftmann |
slightly generalized type class hierarchy concerning unit factors, to allow for lean polynomial normalization
|
file |
diff |
annotate
|
Fri, 30 Dec 2016 18:02:27 +0100 |
haftmann |
more facts on sgn, abs
|
file |
diff |
annotate
|
Sat, 17 Dec 2016 15:22:14 +0100 |
haftmann |
more fine-grained type class hierarchy for div and mod
|
file |
diff |
annotate
|
Sat, 17 Dec 2016 15:22:13 +0100 |
haftmann |
restructured matter on polynomials and normalized fractions
|
file |
diff |
annotate
|
Tue, 18 Oct 2016 18:48:53 +0200 |
haftmann |
suitable logical type class for abs, sgn
|
file |
diff |
annotate
|
Sun, 16 Oct 2016 09:31:05 +0200 |
haftmann |
more standardized theorem names for facts involving the div and mod identity
|
file |
diff |
annotate
|
Sun, 16 Oct 2016 09:31:04 +0200 |
haftmann |
more standardized names
|
file |
diff |
annotate
|
Sun, 16 Oct 2016 09:31:03 +0200 |
haftmann |
added lemma
|
file |
diff |
annotate
|
Wed, 12 Oct 2016 20:38:47 +0200 |
haftmann |
separate type class for arbitrary quotient and remainder partitions
|
file |
diff |
annotate
|
Mon, 26 Sep 2016 07:56:54 +0200 |
haftmann |
syntactic type class for operation mod named after mod;
|
file |
diff |
annotate
|
Mon, 26 Sep 2016 07:56:54 +0200 |
haftmann |
more lemmas
|
file |
diff |
annotate
|
Sun, 18 Sep 2016 17:57:55 +0200 |
haftmann |
more generic algebraic lemmas
|
file |
diff |
annotate
|
Fri, 12 Aug 2016 17:53:55 +0200 |
wenzelm |
more symbols;
|
file |
diff |
annotate
|
Tue, 02 Aug 2016 21:05:34 +0200 |
wenzelm |
misc tuning and modernization;
|
file |
diff |
annotate
|
Tue, 12 Jul 2016 13:55:35 +0200 |
fleury |
sharing simp rules between ordered monoids and rings
|
file |
diff |
annotate
|
Fri, 01 Jul 2016 08:35:15 +0200 |
Manuel Eberl |
More lemmas on Gcd/Lcm
|
file |
diff |
annotate
|
Mon, 20 Jun 2016 21:40:48 +0200 |
wenzelm |
misc tuning and modernization;
|
file |
diff |
annotate
|
Mon, 25 Apr 2016 16:09:26 +0200 |
wenzelm |
eliminated old 'def';
|
file |
diff |
annotate
|
Wed, 16 Mar 2016 13:57:06 +0000 |
paulson |
Contractible sets. Also removal of obsolete theorems and refactoring
|
file |
diff |
annotate
|
Sun, 13 Mar 2016 10:22:46 +0100 |
haftmann |
more theorems on orderings
|
file |
diff |
annotate
|
Tue, 01 Mar 2016 10:36:19 +0100 |
haftmann |
tuned bootstrap order to provide type classes in a more sensible order
|
file |
diff |
annotate
|
Tue, 23 Feb 2016 16:25:08 +0100 |
nipkow |
more canonical names
|
file |
diff |
annotate
|
Fri, 19 Feb 2016 13:40:50 +0100 |
hoelzl |
generalize more theorems to support enat and ennreal
|
file |
diff |
annotate
|
Fri, 12 Feb 2016 16:09:07 +0100 |
hoelzl |
moved more proofs to ordered_comm_monoid_add; introduced strict_ordered_ab_semigroup/comm_monoid_add
|
file |
diff |
annotate
|
Wed, 10 Feb 2016 18:43:19 +0100 |
hoelzl |
Rename ordered_comm_monoid_add to ordered_cancel_comm_monoid_add. Introduce ordreed_comm_monoid_add, canonically_ordered_comm_monoid and dioid. Setup nat, entat and ennreal as dioids.
|
file |
diff |
annotate
|
Thu, 18 Feb 2016 17:53:09 +0100 |
haftmann |
more theorems
|
file |
diff |
annotate
|
Wed, 17 Feb 2016 21:51:57 +0100 |
haftmann |
cleansed junk-producing interpretations for gcd/lcm on nat altogether
|
file |
diff |
annotate
|
Wed, 17 Feb 2016 21:51:57 +0100 |
haftmann |
generalized some lemmas;
|
file |
diff |
annotate
|
Mon, 28 Dec 2015 01:26:34 +0100 |
wenzelm |
prefer symbols for "abs";
|
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
|
Thu, 06 Aug 2015 23:56:48 +0200 |
haftmann |
slight cleanup of lemmas
|
file |
diff |
annotate
|
Sat, 18 Jul 2015 22:58:50 +0200 |
wenzelm |
isabelle update_cartouches;
|
file |
diff |
annotate
|
Wed, 08 Jul 2015 20:19:12 +0200 |
haftmann |
tuned facts
|
file |
diff |
annotate
|
Wed, 08 Jul 2015 14:01:41 +0200 |
haftmann |
avoid explicit definition of the relation of associated elements in a ring -- prefer explicit normalization instead
|
file |
diff |
annotate
|
Wed, 08 Jul 2015 14:01:34 +0200 |
haftmann |
moved normalization and unit_factor into Main HOL corpus
|
file |
diff |
annotate
|
Tue, 30 Jun 2015 13:56:16 +0100 |
paulson |
Useful lemmas. The theorem concerning swapping the variables in a double integral.
|
file |
diff |
annotate
|
Thu, 25 Jun 2015 15:01:42 +0200 |
haftmann |
more theorems
|
file |
diff |
annotate
|
Tue, 23 Jun 2015 16:55:28 +0100 |
paulson |
Amalgamation of the class comm_semiring_1_diff_distrib into comm_semiring_1_cancel. Moving axiom le_add_diff_inverse2 from semiring_numeral_div to linordered_semidom.
|
file |
diff |
annotate
|
Sat, 20 Jun 2015 15:43:36 +0200 |
wenzelm |
avoid suspicious Unicode;
|
file |
diff |
annotate
|
Fri, 19 Jun 2015 07:53:35 +0200 |
haftmann |
separate class for notions specific for integral (semi)domains, in contrast to fields where these are trivial
|
file |
diff |
annotate
|
Fri, 19 Jun 2015 07:53:33 +0200 |
haftmann |
generalized some theorems about integral domains and moved to HOL theories
|
file |
diff |
annotate
|
Fri, 12 Jun 2015 08:53:23 +0200 |
haftmann |
uniform _ div _ as infix syntax for ring division
|
file |
diff |
annotate
|
Mon, 01 Jun 2015 18:59:22 +0200 |
haftmann |
implicit partial divison operation in integral domains
|
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
|
Thu, 02 Apr 2015 11:22:22 +0200 |
haftmann |
semidom contains distributive minus, by convention
|
file |
diff |
annotate
|
Tue, 31 Mar 2015 16:48:48 +0100 |
paulson |
rationalised and generalised some theorems concerning abs and x^2.
|
file |
diff |
annotate
|
Sat, 28 Mar 2015 21:32:48 +0100 |
haftmann |
clarified no_zero_devisors: makes only sense in a semiring;
|
file |
diff |
annotate
|
Sat, 28 Mar 2015 20:43:19 +0100 |
haftmann |
dropped long-outdated comments
|
file |
diff |
annotate
|
Mon, 23 Mar 2015 19:05:14 +0100 |
haftmann |
distributivity of partial minus establishes desired properties of dvd in semirings
|
file |
diff |
annotate
|
Thu, 19 Feb 2015 11:53:36 +0100 |
haftmann |
establish unique preferred fact names
|
file |
diff |
annotate
|
Wed, 18 Feb 2015 22:46:48 +0100 |
haftmann |
eliminated fact duplicates
|
file |
diff |
annotate
|
Sat, 14 Feb 2015 10:24:15 +0100 |
haftmann |
fact consolidation
|
file |
diff |
annotate
|
Mon, 17 Nov 2014 14:55:33 +0100 |
haftmann |
generalized lemmas (particularly concerning dvd) as far as appropriate
|
file |
diff |
annotate
|
Thu, 13 Nov 2014 17:19:52 +0100 |
hoelzl |
import general theorems from AFP/Markov_Models
|
file |
diff |
annotate
|
Sat, 08 Nov 2014 16:53:26 +0100 |
haftmann |
equivalence rules for structures without zero divisors
|
file |
diff |
annotate
|
Sun, 02 Nov 2014 18:21:45 +0100 |
wenzelm |
modernized header uniformly as section;
|
file |
diff |
annotate
|
Fri, 24 Oct 2014 15:07:51 +0200 |
hoelzl |
use NO_MATCH-simproc for distribution rules in field_simps, otherwise field_simps on '(a / (c + d)) * (e + f)' can be non-terminating
|
file |
diff |
annotate
|
Sun, 12 Oct 2014 17:05:34 +0200 |
haftmann |
generalized and consolidated some theorems concerning divisibility
|
file |
diff |
annotate
|