Wed, 10 Jan 2018 15:25:09 +0100 |
nipkow |
ran isabelle update_op on all sources
|
file |
diff |
annotate
|
Wed, 10 Aug 2016 14:50:59 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Mon, 11 Apr 2016 15:26:58 +0200 |
wenzelm |
tuned imports;
|
file |
diff |
annotate
|
Wed, 17 Jun 2015 11:03:05 +0200 |
wenzelm |
isabelle update_cartouches;
|
file |
diff |
annotate
|
Mon, 10 Nov 2014 10:29:19 +0100 |
traytel |
dropped redundant transfer rules (now proved and registered by datatype and plugins)
|
file |
diff |
annotate
|
Sun, 02 Nov 2014 17:20:45 +0100 |
wenzelm |
modernized header;
|
file |
diff |
annotate
|
Tue, 18 Feb 2014 23:03:49 +0100 |
kuncar |
delete or move now not necessary reflexivity rules due to 1726f46d2aa8
|
file |
diff |
annotate
|
Tue, 13 Aug 2013 15:59:22 +0200 |
kuncar |
move Lifting/Transfer relevant parts of Library/Quotient_* to Main
|
file |
diff |
annotate
|
Wed, 05 Jun 2013 15:33:01 +0200 |
kuncar |
transfer rule for listsum
|
file |
diff |
annotate
|
Wed, 15 May 2013 12:10:39 +0200 |
kuncar |
stronger reflexivity prover
|
file |
diff |
annotate
|
Mon, 13 May 2013 13:59:04 +0200 |
kuncar |
better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
|
file |
diff |
annotate
|
Fri, 08 Mar 2013 13:21:52 +0100 |
kuncar |
add [relator_mono] and [relator_distr] rules
|
file |
diff |
annotate
|
Thu, 24 May 2012 14:20:23 +0200 |
kuncar |
prove reflexivity also for the quotient composition relation; reflp_preserve renamed to reflexivity_rule
|
file |
diff |
annotate
|
Wed, 16 May 2012 19:15:45 +0200 |
kuncar |
infrastructure that makes possible to prove that a relation is reflexive
|
file |
diff |
annotate
|
Tue, 15 May 2012 12:07:16 +0200 |
huffman |
transfer rules for many more list constants
|
file |
diff |
annotate
|
Mon, 14 May 2012 17:28:07 +0200 |
huffman |
add transfer rule for constant List.lists
|
file |
diff |
annotate
|
Thu, 26 Apr 2012 12:01:58 +0200 |
kuncar |
use a quot_map theorem attribute instead of the complicated map attribute
|
file |
diff |
annotate
|
Sun, 22 Apr 2012 11:05:04 +0200 |
huffman |
new example theory for quotient/transfer
|
file |
diff |
annotate
|
Sat, 21 Apr 2012 11:21:23 +0200 |
huffman |
add transfer rule for List.set
|
file |
diff |
annotate
|
Sat, 21 Apr 2012 11:04:21 +0200 |
huffman |
remove duplicate of lemma id_transfer
|
file |
diff |
annotate
|
Sat, 21 Apr 2012 07:33:47 +0200 |
huffman |
new transfer package rules and lifting setup for lists
|
file |
diff |
annotate
|
Fri, 20 Apr 2012 18:29:21 +0200 |
kuncar |
hide the invariant constant for relators: invariant_commute infrastracture
|
file |
diff |
annotate
|
Fri, 13 Apr 2012 14:00:26 +0200 |
wenzelm |
updated headers;
|
file |
diff |
annotate
|
Tue, 03 Apr 2012 16:26:48 +0200 |
kuncar |
new package Lifting - initial commit
|
file |
diff |
annotate
|
Fri, 23 Mar 2012 14:20:09 +0100 |
kuncar |
store the relational theorem for every relator
|
file |
diff |
annotate
|
Fri, 24 Feb 2012 22:46:16 +0100 |
haftmann |
explicit is better than implicit
|
file |
diff |
annotate
|
Sat, 10 Dec 2011 13:00:58 +0100 |
huffman |
merged
|
file |
diff |
annotate
|
Fri, 09 Dec 2011 14:14:05 +0100 |
huffman |
remove some duplicate lemmas, simplify some proofs
|
file |
diff |
annotate
|
Fri, 09 Dec 2011 18:07:04 +0100 |
kuncar |
Quotient_Info stores only relation maps
|
file |
diff |
annotate
|
Tue, 30 Nov 2010 15:58:09 +0100 |
haftmann |
more systematic and compact proofs on type relation operators using natural deduction rules
|
file |
diff |
annotate
|
Tue, 09 Nov 2010 14:02:12 +0100 |
haftmann |
fun_rel_def is no simp rule by default
|
file |
diff |
annotate
|
Tue, 19 Oct 2010 12:26:37 +0200 |
bulwahn |
removing something that probably slipped into the Quotient_List theory
|
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
|
Wed, 23 Jun 2010 08:42:41 +0200 |
Cezary Kaliszyk |
Replace 'list_rel' by 'list_all2'; they are equivalent.
|
file |
diff |
annotate
|
Tue, 11 May 2010 07:45:47 +0100 |
Christian Urban |
tuned proof so that no simplifier warning is printed
|
file |
diff |
annotate
|
Thu, 22 Apr 2010 11:55:19 +0200 |
Cezary Kaliszyk |
fun_rel introduction and list_rel elimination for quotient package
|
file |
diff |
annotate
|
Tue, 20 Apr 2010 14:56:58 +0200 |
Cezary Kaliszyk |
respectfullness and preservation of map for identity quotients
|
file |
diff |
annotate
|
Thu, 15 Apr 2010 16:55:12 +0200 |
Cezary Kaliszyk |
Respectfullness and preservation of list_rel
|
file |
diff |
annotate
|
Sun, 14 Mar 2010 14:31:24 +0100 |
wenzelm |
observe standard header format;
|
file |
diff |
annotate
|
Fri, 19 Feb 2010 13:54:19 +0100 |
Cezary Kaliszyk |
Initial version of HOL quotient package.
|
file |
diff |
annotate
|