History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Transfer.thy
Revision Date Author Comments
# e2d96898 27-Jun-2018 immler <none@none>

added lemmas and transfer rules


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

ran isabelle update_op on all sources


# 55f67b56 28-Oct-2016 kuncar <none@none>

a more general relator domain rule for the function type


# bab6845b 03-Oct-2016 haftmann <none@none>

more lemmas

--HG--
extra : rebase_source : f52072de0fdc0fac0b2505569668d385d1ffe93d


# 48473ab7 22-Jun-2016 wenzelm <none@none>

bundle lifting_syntax;


# 1daf8189 13-May-2016 wenzelm <none@none>

eliminated use of empty "assms";


# 6b18406f 16-Feb-2016 traytel <none@none>

make predicator a first-class bnf citizen


# 3487f527 11-Nov-2015 Andreas Lochbihler <none@none>

add various lemmas


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

isabelle update_cartouches;


# 44dc7454 11-Feb-2015 Andreas Lochbihler <none@none>

more transfer rules


# 7a23d6ec 11-Feb-2015 Andreas Lochbihler <none@none>

add parametricity rule for Ex1


# ad953ef3 11-Feb-2015 Andreas Lochbihler <none@none>

add intro and elim rules for right_total


# ef71534e 04-Jan-2015 blanchet <none@none>

tuning


# 07a7056b 19-Dec-2014 desharna <none@none>

Add plugin to generate transfer theorem for primrec and primcorec


# efcf16e5 14-Dec-2014 blanchet <none@none>

renamed theory file

--HG--
rename : src/HOL/Basic_BNF_Least_Fixpoints.thy => src/HOL/Basic_BNF_LFPs.thy


# 75b699bc 05-Dec-2014 kuncar <none@none>

Workaround that allows us to execute lifted constants that have as a return type a datatype containing a subtype


# 23571538 07-Nov-2014 traytel <none@none>

more complete fp_sugars for sum and prod;
tuned;
removed theorem duplicates;
removed obsolete Lifting_{Option,Product,Sum} theories


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

modernized header uniformly as section;


# 8049c47b 29-Oct-2014 wenzelm <none@none>

modernized setup;


# eb1ed55c 25-Sep-2014 desharna <none@none>

generate 'corec_transfer' for codatatypes


# fce1041d 25-Sep-2014 desharna <none@none>

generate 'ctor_rec_transfer' for datatypes


# ee906c73 19-Sep-2014 traytel <none@none>

typo


# a030c224 04-Sep-2014 blanchet <none@none>

tweaked setup for datatype realizer


# 2326a269 01-Sep-2014 blanchet <none@none>

renamed BNF theories

--HG--
rename : src/HOL/BNF_Comp.thy => src/HOL/BNF_Composition.thy
rename : src/HOL/BNF_FP_Base.thy => src/HOL/BNF_Fixpoint_Base.thy
rename : src/HOL/BNF_GFP.thy => src/HOL/BNF_Greatest_Fixpoint.thy
rename : src/HOL/BNF_LFP.thy => src/HOL/BNF_Least_Fixpoint.thy


# d419adf4 21-Jul-2014 Andreas Lochbihler <none@none>

add parametricity lemmas


# 3816e708 27-Jun-2014 blanchet <none@none>

merged two small theory files


# 1ddd04cf 16-Jun-2014 blanchet <none@none>

fixed postprocessing of 'coinduct' formula to obtain right property format (without needless hypotheses)


# 6d2bb8d0 23-Apr-2014 kuncar <none@none>

predicator simplification rules: support also partially specialized types e.g. 'a * nat


# 3532ca39 23-Apr-2014 blanchet <none@none>

qualify name


# f6497c89 11-Apr-2014 kuncar <none@none>

bi_unique and co. rules from the BNF hook must be introduced after bi_unique op= and co. rules are introduced


# e9e8c934 10-Apr-2014 kuncar <none@none>

setup for Transfer and Lifting from BNF; tuned thm names

--HG--
rename : src/HOL/Tools/transfer.ML => src/HOL/Tools/Transfer/transfer.ML


# 15939e27 10-Apr-2014 kuncar <none@none>

abstract Domainp in relator_domain rules => more natural statement of the rule


# 845456ae 10-Apr-2014 kuncar <none@none>

left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)


# 3eabe156 13-Mar-2014 blanchet <none@none>

killed a few 'metis' calls


# b9ba5739 06-Mar-2014 blanchet <none@none>

renamed 'fun_rel' to 'rel_fun'


# bbeeaf3d 28-Feb-2014 traytel <none@none>

load Metis a little later


# 1eaef3ae 26-Feb-2014 kuncar <none@none>

transfer domain rule for special case of functions - was missing


# 40e0ba91 12-Feb-2014 blanchet <none@none>

renamed 'nat_{case,rec}' to '{case,rec}_nat'


# 2312c694 20-Jan-2014 blanchet <none@none>

rationalized lemmas


# 17f4af0c 27-Sep-2013 kuncar <none@none>

new parametricity rules and useful lemmas


# d20e79f0 27-Sep-2013 Andreas Lochbihler <none@none>

add lemmas


# 8c550eac 26-Sep-2013 Andreas Lochbihler <none@none>

add lemmas


# a265459b 13-Aug-2013 kuncar <none@none>

introduce locale with syntax for fun_rel and map_fun and make thus ===> and ---> local


# 63e5edff 10-Jun-2013 huffman <none@none>

implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction


# e63d9dd6 08-Jun-2013 huffman <none@none>

implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>


# 8c36fedb 13-May-2013 kuncar <none@none>

better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal


# c7463a39 12-May-2013 kuncar <none@none>

try to detect assumptions of transfer rules that are in a shape of a transfer rule


# 06f76c96 16-Mar-2013 kuncar <none@none>

fixing transfer tactic - unfold fully identity relation by using relator_eq


# fa22b8b3 13-Feb-2013 haftmann <none@none>

abandoned theory Plain

--HG--
extra : rebase_source : 6f5a395a55e8879386d1f79ab252c6fc2aca7dc5


# 5960ce54 24-Oct-2012 huffman <none@none>

transfer package: more flexible handling of equality relations using is_equality predicate


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

prefer ML_file over old uses;


# 7bae30d6 16-May-2012 kuncar <none@none>

generate abs_eq, use it as a code equation for total quotients; no_abs_code renamed to no_code; added no_code for quotient_type command


# 0f1bc55b 15-May-2012 huffman <none@none>

add transfer rules for nat_rec and funpow


# 2182f6d3 27-Apr-2012 huffman <none@none>

implement transfer tactic with more scalable forward proof methods


# 99b6f075 22-Apr-2012 huffman <none@none>

tuned precedence order of transfer rules

--HG--
extra : rebase_source : fac335be28930b101ac84bd8fb7f88f98bdc10f5


# 92697b81 22-Apr-2012 huffman <none@none>

new example theory for quotient/transfer


# d9f38dea 21-Apr-2012 huffman <none@none>

enable variant of transfer method that proves an implication instead of an equivalence


# 666655c4 20-Apr-2012 huffman <none@none>

add transfer rule for nat_case

--HG--
extra : transplant_source : %26%5B%3A%D7%9B%FA%D9%B6%E95C%04%0E%83%9C%A5%8C%DC8%E2


# 99b9e7e3 20-Apr-2012 huffman <none@none>

uniform naming scheme for transfer rules


# 2fa06ef4 20-Apr-2012 huffman <none@none>

rename 'correspondence' method to 'transfer_prover'


# 1ad97ca5 20-Apr-2012 huffman <none@none>

add secondary transfer rule for universal quantifiers on non-bi-total relations


# 791ae3a6 20-Apr-2012 huffman <none@none>

add transfer rule for 'id'


# a3bc0689 20-Apr-2012 huffman <none@none>

make correspondence tactic more robust by replacing lhs with schematic variable before applying intro rules


# d74af506 19-Apr-2012 huffman <none@none>

add transfer rule for Let


# 680b0253 17-Apr-2012 huffman <none@none>

make transfer method more deterministic by using SOLVED' on some subgoals

--HG--
extra : rebase_source : 3ed8e05dc4c7ebb812ea7cdcdd0b9bbe2de94ebd


# 985992de 17-Apr-2012 huffman <none@none>

add theory data for relator identity rules;
preprocess transfer rules generated by lift_definition using relator rules

--HG--
extra : transplant_source : %0C%BB%B3H%AB%A7%25/H%DF%AE%0E%AF%8B%F83-%9AK%06


# 0a08d4aa 04-Apr-2012 huffman <none@none>

add bounded quantifier constant transfer_bforall, whose definition is unfolded after transfer


# f0c3385b 03-Apr-2012 huffman <none@none>

new transfer proof method