History log of /seL4-l4v-master/isabelle/src/HOL/Tools/Lifting/lifting_def_code_dt.ML
Revision Date Author Comments
# 14c7fb8f 09-Aug-2019 wenzelm <none@none>

formal position for PThm nodes;


# 44401f83 04-Jun-2019 wenzelm <none@none>

proper context;


# 0c041064 04-Jun-2019 wenzelm <none@none>

misc tuning and clarification, notably wrt. flow of context;


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

isabelle update -u control_cartouches;


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

isabelle update -u control_cartouches;


# f413faf7 23-Feb-2018 wenzelm <none@none>

tuned signature;


# e1a2167e 05-Jun-2017 haftmann <none@none>

avoid Local_Theory.reset in application space

--HG--
extra : rebase_source : 085dbafb40406dfe49ff89a0341696228dcbd526


# bee57ad5 23-Jun-2016 wenzelm <none@none>

tuned signature;


# c71812c7 21-Jun-2016 wenzelm <none@none>

tuned;


# 3dba35c1 27-May-2016 wenzelm <none@none>

tuned proofs, to allow unfold_abs_def;


# ef845594 17-Apr-2016 wenzelm <none@none>

clarified signature;


# 5dc803d8 13-Apr-2016 wenzelm <none@none>

eliminated "xname" and variants;


# 361a1e00 04-Mar-2016 wenzelm <none@none>

tuned signature;


# 369e4785 13-Dec-2015 wenzelm <none@none>

more general types Proof.method / context_tactic;
proper context for Method.insert_tac;
tuned;


# 55ef7203 17-Oct-2015 wenzelm <none@none>

tuned signature;


# 839d9ae3 26-Jul-2015 wenzelm <none@none>

updated to infer_instantiate;


# 62ae9c62 18-Jul-2015 wenzelm <none@none>

prefer tactics with explicit context;


# dbbe37ca 15-Jul-2015 traytel <none@none>

{r,e,d,f}tac with proper context in BNF


# b57e1113 06-Jul-2015 wenzelm <none@none>

tuned;


# bfa1f692 15-Jun-2015 wenzelm <none@none>

tuned;


# db484122 07-Jun-2015 wenzelm <none@none>

tuned signature;


# b74c761c 03-May-2015 wenzelm <none@none>

make SML/NJ more happy;


# cd9a1930 02-May-2015 kuncar <none@none>

handle error messages also in after_qed


# 6c62572f 02-May-2015 kuncar <none@none>

reorder some steps in the construction to support mutual datatypes


# 7327e9b1 02-May-2015 kuncar <none@none>

more readable error message if some types do not correspond to sort constraints of the datatype


# c4a952b9 02-May-2015 kuncar <none@none>

better precomputing


# 351bf560 02-May-2015 kuncar <none@none>

equivalence in code_dt data structure must respect both rty and qty


# cd379f20 02-May-2015 kuncar <none@none>

don't use the human-readable version of the rsp thm as a goal in the ML interface (there is no formal definition of its statement); make tactics more robust wrt. predicates in predicators; tuned


# 11e5f72a 13-Apr-2015 kuncar <none@none>

go back to the complicated code equation registration (because of type classes) that was lost in 922586b1bc87; make it even more hackish to get which code equation was used


# 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