History log of /seL4-l4v-master/isabelle/src/HOL/Transitive_Closure.thy
Revision Date Author Comments
# 043c3b16 18-Jan-2020 traytel <none@none>

new examples of BNF lifting across quotients using a new theory of confluence,
which simplifies the relator subdistributivity proof obligation
(a few new useful notions were added to HOL;
notably the symmetric and equivalence closures of a relation)


# c56a85fc 23-Sep-2019 paulson <lp15@cam.ac.uk>

More type class generalisations. Note that linorder_antisym_conv1 and linorder_antisym_conv2 no longer exist.


# e60cf64d 06-Jan-2019 wenzelm <none@none>

isabelle update -u path_cartouches;


# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# a4bab154 04-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# e01498ae 10-Nov-2018 haftmann <none@none>

replaced some ancient ASCII syntax


# 685c0eec 12-Jul-2018 paulson <lp15@cam.ac.uk>

de-applying (mostly Set_Interval)


# 43b1852b 16-Jun-2018 nipkow <none@none>

more simp


# 5128613b 16-Jun-2018 nipkow <none@none>

moved lemmas from AFP


# 63ba3fbf 25-Feb-2018 wenzelm <none@none>

more abbrevs;


# f5796e6d 14-Feb-2018 wenzelm <none@none>

more symbols;


# a7ccdf43 10-Jan-2018 nipkow <none@none>

ran isabelle update_op on all sources


# 45a0e905 05-Aug-2016 wenzelm <none@none>

misc tuning and modernization;


# 1f8ba5d4 06-Jul-2016 wenzelm <none@none>

misc tuning and modernization;


# 1af22de0 12-Apr-2016 wenzelm <none@none>

tuned;


# 6688eecc 17-Feb-2016 haftmann <none@none>

prefer abbreviations for compound operators INFIMUM and SUPREMUM


# 4216bc36 07-Jan-2016 wenzelm <none@none>

more uniform treatment of package internals;


# 0bfb73b6 28-Dec-2015 wenzelm <none@none>

former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";


# 0df376fc 07-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 2ceb4cc9 14-Nov-2015 wenzelm <none@none>

option "inductive_defs" controls exposure of def and mono facts;


# 18551fee 13-Oct-2015 haftmann <none@none>

prod_case as canonical name for product type eliminator


# 607ae3e3 09-Oct-2015 wenzelm <none@none>

discontinued specific HTML syntax;


# df44ab4c 27-Aug-2015 haftmann <none@none>

standardized some occurences of ancient "split" alias

--HG--
extra : rebase_source : 706ba501d5c0596a2bde6e46d42aa8464a91ede5


# 1901affb 18-Jul-2015 wenzelm <none@none>

isabelle update_cartouches;


# 2a31d0b7 07-Jul-2015 hoelzl <none@none>

add monotonicity rule for rtranclp


# 794edf80 02-Nov-2014 wenzelm <none@none>

modernized header uniformly as section;


# c9fd506f 21-Jun-2014 nipkow <none@none>

r_into_(r)trancl should not be [simp]: helps little and comlicates some AFP proofs


# c817ea9d 21-Jun-2014 nipkow <none@none>

added [simp]


# 3b0b1891 06-Jun-2014 nipkow <none@none>

added lemmas


# 9c548546 22-Mar-2014 wenzelm <none@none>

more antiquotations;


# 04523a1c 19-Feb-2014 blanchet <none@none>

moved 'primrec' up (for real this time) and removed temporary 'old_primrec'


# 3154df20 17-Feb-2014 blanchet <none@none>

renamed old 'primrec' to 'old_primrec' (until the new 'primrec' can be moved above 'Nat' in the theory dependencies)


# aff8c6a4 12-Feb-2014 blanchet <none@none>

adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
* * *
more transition of 'xxx_rec' to 'rec_xxx' and same for case
* * *
compile
* * *
'rename_tac's to avoid referring to generated names
* * *
more robust scripts with 'rename_tac'
* * *
'where' -> 'of'
* * *
'where' -> 'of'
* * *
renamed 'xxx_rec' to 'rec_xxx'


# 28ac67aa 12-Nov-2013 hoelzl <none@none>

add acyclicI_order


# 0928b2db 18-Apr-2013 wenzelm <none@none>

simplifier uses proper Proof.context instead of historic type simpset;


# 052f6f87 23-Dec-2012 nipkow <none@none>

renamed and added lemmas


# e3227796 22-Aug-2012 wenzelm <none@none>

prefer ML_file over old uses;


# 46f8e6d2 16-Apr-2012 Christian Sternagel <none@none>

duplicate "relpow" facts for "relpowp" (to emphasize that both worlds exist and obtain better search results with "find_theorems")


# 55e11b0d 03-Apr-2012 griff <none@none>

renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")


# 190d3852 30-Mar-2012 haftmann <none@none>

power on predicate relations


# 94314ed4 01-Mar-2012 haftmann <none@none>

more fundamental pred-to-set conversions, particularly by means of inductive_set; associated consolidation of some theorem names (c.f. NEWS)


# 484c9d58 24-Feb-2012 haftmann <none@none>

moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy

--HG--
extra : rebase_source : ed15629634477aff0a8efea30547f496c70907ad


# 37822d49 23-Feb-2012 haftmann <none@none>

moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy


# 76a8769b 30-Jan-2012 bulwahn <none@none>

renaming all lemmas with name rel_pow to relpow


# 17ae6b1d 30-Jan-2012 bulwahn <none@none>

adding code generation for relpow by copying the ideas for code generation of funpow


# 4379bd6d 27-Jan-2012 bulwahn <none@none>

new code equation for ntrancl that allows computation of the transitive closure of sets on infinite types as well


# 26ada052 01-Jan-2012 haftmann <none@none>

cleanup of code declarations

--HG--
extra : rebase_source : 7376929a640011e27309be6654ccf370df37e60a


# 6e9d7f07 24-Dec-2011 haftmann <none@none>

tuned layout


# a495a026 20-Nov-2011 wenzelm <none@none>

eliminated obsolete "standard";


# ad002749 16-Oct-2011 haftmann <none@none>

tuned type annnotation


# 5d6d046e 13-Oct-2011 haftmann <none@none>

avoid very specific code equation for card; corrected spelling

--HG--
extra : rebase_source : 7a43ff22845a7caa93989e5f5ab5908190833404


# c5612a1a 13-Oct-2011 haftmann <none@none>

bouned transitive closure

--HG--
extra : rebase_source : 3d0df473619b9c72b32a96ed4951a34dd2ad6c82


# 09ec04b4 13-Oct-2011 haftmann <none@none>

moved acyclic predicate up in hierarchy

--HG--
extra : rebase_source : 4c9a0c3c1dd3de32826493a20016e209648a4e47


# 0f6d12b7 13-Oct-2011 haftmann <none@none>

modernized definitions

--HG--
extra : rebase_source : d50ecbd4a46b11ec1f49c3eb54ad2ee86a8981ce


# 77fe7d87 03-Oct-2011 bulwahn <none@none>

adding lemma about rel_pow in Transitive_Closure for executable equation of the (refl) transitive closure


# 15635718 13-Sep-2011 huffman <none@none>

tuned proofs


# ad9e459c 11-Sep-2011 nipkow <none@none>

new fastforce replacing fastsimp - less confusing name


# 9c72c6e0 29-Jun-2011 wenzelm <none@none>

simplified/unified Simplifier.mk_solver;


# 14ffc3e9 13-May-2011 wenzelm <none@none>

clarified map_simpset versus Simplifier.map_simpset_global;


# 64269ee0 16-Mar-2011 nipkow <none@none>

added lemmas


# 47bb2a89 21-Feb-2011 blanchet <none@none>

renamed "nitpick\_def" to "nitpick_unfold" to reflect its new semantics


# 5b59da77 13-Sep-2010 nipkow <none@none>

renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI


# bb8268b1 07-Sep-2010 nipkow <none@none>

expand_fun_eq -> ext_iff
expand_set_eq -> set_ext_iff
Naming in line now with multisets


# b6d43d5c 01-Jul-2010 haftmann <none@none>

qualified constants Set.member and Set.Collect


# 42aff2ea 09-Jun-2010 haftmann <none@none>

tuned quotes, antiquotations and whitespace


# aaaa7964 18-Feb-2010 huffman <none@none>

get rid of many duplicate simp rule warnings


# 37749a72 27-Jan-2010 haftmann <none@none>

lemma Image_closed_trancl


# 0d6997ba 10-Jan-2010 berghofe <none@none>

Tuned some proofs; nicer case names for some of the induction / cases rules.


# b0676530 24-Nov-2009 blanchet <none@none>

removed "nitpick_def" attributes from (r)trancl(p), since "Nitpick.thy" overrides these


# 6cc60f7d 13-Nov-2009 krauss <none@none>

a few lemmas for point-free reasoning about transitive closure


# d417f500 09-Oct-2009 haftmann <none@none>

simplified proof


# 3641ced1 06-Oct-2009 haftmann <none@none>

inf/sup1/2_iff are mere duplicates of underlying definitions: dropped


# 4c81b643 18-Sep-2009 haftmann <none@none>

be more cautious wrt. simp rules: sup1_iff, sup2_iff, inf1_iff, inf2_iff, SUP1_iff, SUP2_iff, INF1_iff, INF2_iff are no longer simp by default


# 263e675f 27-Jul-2009 krauss <none@none>

"more standard" argument order of relation composition (op O)


# f65d489e 26-Jul-2009 wenzelm <none@none>

replaced old METAHYPS by FOCUS;
eliminated homegrown SUBGOAL combinator -- beware of exception Subscript in body;
modernized functor names;
minimal tuning of sources;
reactivated dead quasi.ML (ever used?);


# 19f01caa 09-Jul-2009 krauss <none@none>

move rel_pow_commute: "R O R ^^ n = R ^^ n O R" to Transitive_Closure


# ea5b338b 17-Jun-2009 nipkow <none@none>

rtrancl lemmas


# bc04886a 11-Jun-2009 bulwahn <none@none>

added lemma


# 5e941416 11-Jun-2009 bulwahn <none@none>

added lemma


# 5fbe34a5 01-Jun-2009 nipkow <none@none>

new lemma


# 13866ee3 24-Apr-2009 haftmann <none@none>

funpow and relpow with shared "^^" syntax


# ceaab00c 20-Apr-2009 haftmann <none@none>

power operation on functions in theory Nat; power operation on relations in theory Transitive_Closure


# b1258973 16-Mar-2009 wenzelm <none@none>

simplified method setup;


# 77d6b267 13-Mar-2009 wenzelm <none@none>

unified type Proof.method and pervasive METHOD combinators;


# 121e82fb 04-Mar-2009 blanchet <none@none>

Merge.


# bb2d682e 02-Mar-2009 nipkow <none@none>

name changes


# 9ca47f79 26-Feb-2009 berghofe <none@none>

Fixed nonexhaustive match problem in decomp, to make it fail more gracefully
in case assumptions are not of the form (Trueprop $ ...).


# 73d9a35c 21-Jan-2009 haftmann <none@none>

changed import hierarchy


# 9f177be5 07-May-2008 berghofe <none@none>

- Function dec in Trancl_Tac must eta-contract relation before calling
decr, since it is now a function and could therefore be in eta-expanded form
- The trancl prover now does more eta-contraction itself, so eta-contraction
is no longer necessary in Tranclp_tac.


# 13b177d7 19-Mar-2008 wenzelm <none@none>

more antiquotations;
eliminated change_claset/simpset;


# 6cef3e0f 14-Mar-2008 nipkow <none@none>

Added lemmas


# 6fbba864 28-Feb-2008 wenzelm <none@none>

rtranclp_induct, tranclp_induct: added case_names;
tuned proofs;


# 7be5f862 27-Feb-2008 wenzelm <none@none>

rtranclE, tranclE: tuned statement, added case_names;


# cf72fafb 13-Nov-2007 berghofe <none@none>

Removed some case_names and consumes attributes that are now no longer
needed due to changes in the to_pred and to_set attributes.


# ef361cf1 05-Nov-2007 kleing <none@none>

tranclD2 (tranclD at the other end) + trancl_power


# 67ccb1e5 11-Jul-2007 berghofe <none@none>

rtrancl and trancl are now defined using inductive_set.


# e1e12128 09-Mar-2007 haftmann <none@none>

stepping towards uniform lattice theory development in HOL


# 1daf9028 07-Feb-2007 berghofe <none@none>

Adapted to new inductive definition package.


# c41552bd 24-Jan-2007 paulson <none@none>

some new lemmas


# 21214e74 17-Jan-2007 paulson <none@none>

induction rules for trancl/rtrancl expressed using subsets


# 0da20efc 29-Nov-2006 wenzelm <none@none>

simplified method setup;
reactivated dead code;


# cd65d9bc 16-Nov-2006 wenzelm <none@none>

more robust syntax for definition/abbreviation/notation;


# cbb1a051 07-Nov-2006 wenzelm <none@none>

renamed 'const_syntax' to 'notation';


# 1e731d3a 26-Sep-2006 krauss <none@none>

Changed precedence of "op O" (relation composition) from 60 to 75.


# 61bd82ad 16-May-2006 wenzelm <none@none>

tuned concrete syntax -- abbreviation/const_syntax;


# d1dc012d 12-May-2006 nipkow <none@none>

added lemma in_measure


# ca6e4a30 09-Mar-2006 huffman <none@none>

added many simple lemmas


# d2b0060d 08-Dec-2005 wenzelm <none@none>

tuned proofs;


# 3deee062 17-Oct-2005 wenzelm <none@none>

change_claset/simpset;


# 0789ab36 22-Sep-2005 nipkow <none@none>

renamed rules to iprover


# c4406fb7 21-Jun-2005 kleing <none@none>

lemma, equation between rtrancl and trancl


# a7060872 17-Jun-2005 haftmann <none@none>

migrated theory headers to new format


# 9f1ea5d9 21-Apr-2005 wenzelm <none@none>

superceded by Pure.thy and CPure.thy;


# b55c62f0 28-Feb-2005 paulson <none@none>

unfold theorems for trancl and rtrancl


# 3dffd254 13-Feb-2005 skalberg <none@none>

Deleted Library.option type.


# 0fe1d442 18-Aug-2004 nipkow <none@none>

import -> imports


# e61c8d7d 16-Aug-2004 nipkow <none@none>

New theory header syntax.


# dd412ee2 02-Aug-2004 ballarin <none@none>

Documentation added; minor improvements.


# 1a1a40cb 26-Jul-2004 ballarin <none@none>

New prover for transitive and reflexive-transitive closure of relations.
- Code in Provers/trancl.ML
- HOL: Simplifier set up to use it as solver


# cd257618 14-Apr-2004 kleing <none@none>

use more symbols in HTML output


# 1ff26745 21-Feb-2004 nipkow <none@none>

Transitive_Closure: added consumes and case_names attributes
Isar: fixed parameter name handling in simulatneous induction
which I had not done properly 2 years ago.


# 29c20de7 19-Feb-2004 ballarin <none@none>

Efficient, graph-based reasoner for linear and partial orders.
+ Setup as solver in the HOL simplifier.


# 55f6b81a 26-Jan-2004 schirmer <none@none>

* Support for raw latex output in control symbols: \<^raw...>
* Symbols may only start with one backslash: \<...>. \\<...> is no longer
accepted by the scanner.
- Adapted some Isar-theories to fit to this policy


# eade7171 04-Jan-2004 nipkow <none@none>

undid split_comp_eq[simp] because it leads to nontermination together with split_def!


# b79b3996 26-Sep-2003 paulson <none@none>

misc tidying


# 7aa30ca2 17-Mar-2003 nipkow <none@none>

just a few mods to a few thms


# df6362b8 27-Nov-2002 berghofe <none@none>

Replaced some blasts by rules.


# aa4aa83c 13-Nov-2002 berghofe <none@none>

Transitive closure is now defined inductively as well.


# 74fc2075 25-Feb-2002 wenzelm <none@none>

clarified syntax of ``long'' statements: fixes/assumes/shows;


# 1c57f335 21-Jan-2002 berghofe <none@none>

Made some proofs constructive.


# ec66e0a1 09-Jan-2002 wenzelm <none@none>

converted theory Transitive_Closure;


# 89c4958e 20-Dec-2001 nipkow <none@none>

renamed rtrancl_into_rtrancl2 to converse_rtrancl_into_rtrancl


# db21bad2 09-Dec-2001 kleing <none@none>

setup [trans] rules for calculational Isar reasoning


# 18cd56b5 22-May-2001 berghofe <none@none>

Transitive closure is now defined via "inductive".


# 1172ad83 13-Feb-2001 paulson <none@none>

a new theorem from Bryan Ford


# 48e2f73b 09-Feb-2001 wenzelm <none@none>

tuned;


# 543068b0 09-Feb-2001 wenzelm <none@none>

unsymbolized;
tuned;


# 225b016b 29-Jan-2001 nipkow <none@none>

Moved some thms from Transitive_ClosureTr.ML to Transitive_Closure.thy


# 8a679c39 25-Jan-2001 wenzelm <none@none>

Transitive_Closure turned into new-style theory;


# a81dee75 08-Jan-2001 wenzelm <none@none>

syntax (xsymbols);


# a7873168 01-Dec-2000 wenzelm <none@none>

superscripts: syntax (latex);


# 1af90e23 25-Oct-2000 wenzelm <none@none>

more "xsymbols" syntax;


# 322ec07c 12-Oct-2000 nipkow <none@none>

*** empty log message ***