History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Quotient.thy
Revision Date Author Comments
# 22929640 11-Jul-2018 paulson <lp15@cam.ac.uk>

de-applying (mostly Quotient)


# 0277d8a8 11-Jul-2018 paulson <lp15@cam.ac.uk>

de-applying


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

ran isabelle update_op on all sources


# c7cc1919 26-Nov-2017 wenzelm <none@none>

more symbols;


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

bundle lifting_syntax;


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

isabelle update_cartouches -c -t;


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

isabelle update_cartouches;


# 37b9ab28 22-Nov-2014 wenzelm <none@none>

named_theorems: multiple args;


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

modernized header uniformly as section;


# 8b2e1ce1 16-Aug-2014 wenzelm <none@none>

updated to named_theorems;
modernized setup;


# 713cd402 13-Mar-2014 nipkow <none@none>

enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions

--HG--
extra : rebase_source : 4103bf02b2df95e1e84808f766f131292beef893


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

renamed 'fun_rel' to 'rel_fun'


# 355cccc4 26-Dec-2013 haftmann <none@none>

prefer ephemeral interpretation over interpretation in proof contexts;
prefer context begin ... end blocks for often-occuring assumptions;
slightly more complete interpretations into abstract algebraic structures for gcd/lcm


# f55a6e4d 21-Nov-2013 blanchet <none@none>

rationalize imports


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

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


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

abandoned theory Plain

--HG--
extra : rebase_source : 6f5a395a55e8879386d1f79ab252c6fc2aca7dc5


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

prefer ML_file over old uses;


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

move definition of set_rel into Library/Quotient_Set.thy


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

tuned lemmas (v)image_id;
removed duplicate of vimage_id

--HG--
extra : rebase_source : 9178db2e0f900cdeab723f13b8c0d5fc45786a95


# b5a49119 18-Apr-2012 huffman <none@none>

move constant 'Respects' into Lifting.thy;
add quantifier transfer rules for quotients


# f928efd2 15-Apr-2012 haftmann <none@none>

centralized enriched_type declaration, thanks to in-situ available Isar commands

--HG--
extra : rebase_source : ea8947ffa8bb301d674c472c3427994b31c4c458


# cedccc64 04-Apr-2012 kuncar <none@none>

connect the Quotient package to the Lifting package


# fe6190cb 04-Apr-2012 kuncar <none@none>

support non-open typedefs; define cr_rel in terms of a rep function for typedefs


# a2076df5 03-Apr-2012 kuncar <none@none>

new package Lifting - initial commit


# c03a8511 03-Apr-2012 griff <none@none>

dropped abbreviation "pred_comp"; introduced infix notation "P OO Q" for "relcompp P Q"


# 23c06d7b 23-Mar-2012 kuncar <none@none>

hide invariant constant


# 870593bf 15-Mar-2012 wenzelm <none@none>

declare command keywords via theory header, including strict checking outside Pure;


# 9986980f 15-Mar-2012 wenzelm <none@none>

declare minor keywords via theory header;


# 52a77b75 14-Feb-2012 wenzelm <none@none>

simplified use of tacticals;


# 5a4d46ec 23-Mar-2012 kuncar <none@none>

generation of a code certificate from a respectfulness theorem for constants lifted by the quotient_definition command & setup_lifting command: setups Quotient infrastructure from a typedef theorem


# 549cca3b 23-Mar-2012 kuncar <none@none>

store the relational theorem for every relator


# 30cfef34 23-Mar-2012 kuncar <none@none>

respectfulness theorem has to be proved if a new constant is lifted by quotient_definition


# c8373369 24-Dec-2011 haftmann <none@none>

treatment of type constructor `set`


# fbb710bf 09-Dec-2011 kuncar <none@none>

Quotient_Info stores only relation maps


# 0ef878e6 07-Dec-2011 Christian Urban <urbanc@in.tum.de>

added a specific tactic and method that deal with partial equivalence relations


# 63baa0b0 29-Nov-2011 wenzelm <none@none>

more conventional file name;

--HG--
rename : src/HOL/Tools/Quotient/quotient_typ.ML => src/HOL/Tools/Quotient/quotient_type.ML


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

tuned proofs


# c8a8b241 26-Aug-2011 haftmann <none@none>

avoid intermixing set and predicates; dropped lemmas mem_rsp and mem_prs (now in Quotient_Set.thy)


# 50ebd0cd 22-Aug-2011 Cezary Kaliszyk <kaliszyk@in.tum.de>

Quotient Package: some infrastructure for lifting inside sets


# 2304bb0b 16-Aug-2011 haftmann <none@none>

avoid Collect_def in proof


# 83a642c7 15-Aug-2011 Cezary Kaliszyk <kaliszyk@in.tum.de>

Quotient Package: make quotient_type work with separate set type


# 10eb7fb0 15-May-2011 wenzelm <none@none>

simplified/unified method_setup/attribute_setup;


# 69d1859b 14-Apr-2011 blanchet <none@none>

use old Skolemizer for Metis call that requires high unification bound (around 100) with the new Skolemizer


# 6b0b29ec 13-Mar-2011 wenzelm <none@none>

tuned headers;


# 44036fcf 07-Jan-2011 wenzelm <none@none>

more standard package setup;


# 9d87b269 29-Nov-2010 haftmann <none@none>

reorienting iff in Quotient_rel prevents simplifier looping;
lemma QuotientI;
tuned theory text


# b623a392 28-Nov-2010 haftmann <none@none>

moved generic definitions about (partial) equivalence relations from Quotient to Equiv_Relations;
moved generic definitions about relations from Quotient.thy to Predicate;
consistent use of R rather than E for relations;
more natural deduction rules


# 0ba310a7 19-Nov-2010 haftmann <none@none>

generalized type


# 172e431c 18-Nov-2010 haftmann <none@none>

map_fun combinator in theory Fun


# 1343acec 09-Nov-2010 haftmann <none@none>

type annotations in specifications; fun_rel_def is no simp rule by default; slightly changed fun_map_def; more on predicates on relation functions; proper HOL equations in definitions


# cfd108c9 18-Oct-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Quotient package: partial equivalence introduction


# a383962e 04-Oct-2010 blanchet <none@none>

remove needless Metis facts


# 37d247fe 04-Oct-2010 blanchet <none@none>

move Metis into Plain

--HG--
rename : src/HOL/Tools/Sledgehammer/metis_reconstruct.ML => src/HOL/Tools/Metis/metis_reconstruct.ML
rename : src/HOL/Tools/Sledgehammer/metis_tactics.ML => src/HOL/Tools/Metis/metis_tactics.ML
rename : src/HOL/Tools/Sledgehammer/metis_translate.ML => src/HOL/Tools/Metis/metis_translate.ML


# d87e74ba 24-Sep-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

quotient package: respectfulness and preservation of identity.


# 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


# df213d75 30-Aug-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Quotient Package: added respectfulness and preservation lemmas for mem.


# 38c86d01 28-Aug-2010 Christian Urban <urbanc@in.tum.de>

quotient package: lemmas to be lifted and descended can be pre-simplified


# ab2bef15 24-Aug-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Quotient Package / lemma for regularization of bex1_rel for equivalence relations


# 68e44906 10-Aug-2010 Christian Urban <urbanc@in.tum.de>

deleted duplicate lemma


# 44656fed 27-Jul-2010 wenzelm <none@none>

use file names relative to master directory of theory source -- Proof General can now handle that due to the ThyLoad.add_path deception (cf. 3ceccd415145);


# 402fd610 28-Jun-2010 Christian Urban <urbanc@in.tum.de>

separated the lifting and descending procedures in the quotient package


# 320b0406 28-Jun-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Quotient package reverse lifting


# fe0c75d5 23-Jun-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Quotient package now uses Partial Equivalence instead place of equivalence


# b0c56ea9 21-May-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Let rsp and prs in fun_rel/fun_map format


# 1d0c8196 22-Apr-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

fun_rel introduction and list_rel elimination for quotient package


# 38878c5e 20-Apr-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

respectfullness and preservation of function composition


# 5815b59f 13-Apr-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

add If respectfullness and preservation to Quotient package database


# b6714212 12-Apr-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Changed the type of Quot_True, so that it is an HOL constant.


# eaf6f9f8 17-Mar-2010 blanchet <none@none>

renamed "ATP_Linkup" theory to "Sledgehammer"

--HG--
rename : src/HOL/ATP_Linkup.thy => src/HOL/Sledgehammer.thy


# c266a1be 22-Feb-2010 huffman <none@none>

proper header and subsection headings


# 46e8c65f 19-Feb-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

quote the constant and theorem name with @{text}


# d051685e 19-Feb-2010 Cezary Kaliszyk <kaliszyk@in.tum.de>

Initial version of HOL quotient package.