Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
ML_Antiquote.value;
2008-06-24, by wenzelm
added isaantiqopen/close;
2008-06-24, by wenzelm
Logic.all/mk_equals/mk_implies;
2008-06-23, by wenzelm
moved implies to logic.ML;
2008-06-23, by wenzelm
added all, is_all;
2008-06-23, by wenzelm
Logic.implies;
2008-06-23, by wenzelm
Logic.is_all;
2008-06-23, by wenzelm
Term.all;
2008-06-23, by wenzelm
Logic.all/mk_equals/mk_implies;
2008-06-23, by wenzelm
session name: empty for Pure and by default;
2008-06-23, by wenzelm
induct_tac: allow omission of arguments;
2008-06-23, by wenzelm
info: default name is "", not "Pure";
2008-06-23, by wenzelm
moved src/HOL/Tools/induct_tacs.ML to src/Tools/induct_tacs.ML;
2008-06-23, by wenzelm
removed obsolete dest_concls;
2008-06-23, by wenzelm
induct_tac: mutual rules work as for method "induct";
2008-06-23, by wenzelm
tuned get_inductT: *all* rules for missing instantiation;
2008-06-23, by wenzelm
induct_tac: infer mutual rule from types, as for proper induct method;
2008-06-23, by wenzelm
induct_tac/case_tac: nested tuples are split as expected;
2008-06-23, by wenzelm
induct_tac: old conjunctive rules no longer supported;
2008-06-23, by wenzelm
updated generated file;
2008-06-23, by wenzelm
induct_tac: rule is inferred from types;
2008-06-23, by wenzelm
cleaned up some proofs;
2008-06-22, by huffman
use new-style abbreviation/notation for fix syntax
2008-06-22, by huffman
import_export_proof: simplified thm definition -- PureThy.name_thm does the job;
2008-06-21, by wenzelm
added query_type/const/class (meta data);
2008-06-21, by wenzelm
the_tags: explicit error message;
2008-06-21, by wenzelm
activate_context: strict the_context, no fallback on theory context;
2008-06-21, by wenzelm
remove unused constant liftpair
2008-06-20, by huffman
simplify profinite class axioms
2008-06-20, by huffman
clean up and rename some profinite lemmas
2008-06-20, by huffman
move at-sml-dev-e to macbroy23
2008-06-20, by isatest
replace SetPcpo.thy with Cset.thy
2008-06-20, by huffman
updated for 2008;
2008-06-20, by wenzelm
(removed non-present change)
2008-06-20, by haftmann
explicit thm context for error messages
2008-06-20, by haftmann
using tages to find theory names
2008-06-20, by haftmann
type constructors now with markup
2008-06-20, by haftmann
fixed bind error for malformed primrec specifications
2008-06-20, by haftmann
DatatypeProp.make_distincts: only one half of each symmetric pair is constructed
2008-06-20, by haftmann
streamlined definitions
2008-06-20, by haftmann
moved Float.thy to Library
2008-06-20, by haftmann
removed SetPcpo.thy and cpo instance for type bool;
2008-06-20, by huffman
moved Abs_image to Typedef.thy; prove finite_UNIV outside the locale
2008-06-20, by huffman
add lemma Abs_image
2008-06-20, by huffman
added some lemmas; reorganized into sections; tuned proofs
2008-06-20, by huffman
added some lemmas; tuned proofs
2008-06-20, by huffman
tuned
2008-06-20, by huffman
replace less_lift with flat_less_iff
2008-06-20, by huffman
tweak lemmas adm_all and adm_ball
2008-06-20, by huffman
move lemmas into locales;
2008-06-19, by huffman
add lemmas take_chain_less and take_chain_le
2008-06-19, by huffman
disposed Sign.read_typ etc;
2008-06-19, by wenzelm
renamed is_abbrev_mode to abbrev_mode;
2008-06-19, by wenzelm
ProofContext.abbrev_mode;
2008-06-19, by wenzelm
moved get_sort to Isar/proof_context.ML;
2008-06-19, by wenzelm
tuned signature;
2008-06-19, by wenzelm
private add_used (from drule.ML);
2008-06-19, by wenzelm
Variable.declare_typ;
2008-06-19, by wenzelm
added declare_typ;
2008-06-19, by wenzelm
moved add_used to Isar/rule_insts.ML;
2008-06-19, by wenzelm
export read_typ/cert_typ -- version with regular context operations;
2008-06-19, by wenzelm
export read_typ/cert_typ -- version with regular context operations;
2008-06-19, by wenzelm
tuned signature;
2008-06-19, by wenzelm
removed duplicate of DatatypePackage.read_typ;
2008-06-19, by wenzelm
add lemma cfcomp_LAM
2008-06-19, by huffman
add_abbrev: check tfrees of rhs, not tvars (addresses a lapse introduced in 1.65);
2008-06-19, by wenzelm
slightly tuned
2008-06-19, by urbanc
generalized induct_scheme method to prove conditional induction schemes.
2008-06-19, by krauss
add lemma iterate_iterate
2008-06-19, by huffman
* Disposed old term read functions;
2008-06-18, by wenzelm
replace preorder class with locale
2008-06-18, by huffman
add lemma compact_imp_principal to locale ideal_completion
2008-06-18, by huffman
added type_constraint (formerly in type_infer.ML, which is now loaded later);
2008-06-18, by wenzelm
TypeExt.type_constraint;
2008-06-18, by wenzelm
simplified TypeInfer.infer_types;
2008-06-18, by wenzelm
improved error output -- variant/mark bounds;
2008-06-18, by wenzelm
load type_infer.ML after Syntax module;
2008-06-18, by wenzelm
eliminated old Sign.read_term/Thm.read_cterm etc.;
2008-06-18, by wenzelm
moved ProofContext.pretty_proof to ProofSyntax.pretty_proof;
2008-06-18, by wenzelm
export transfer_syntax;
2008-06-18, by wenzelm
moved ProofContext.pretty_proof to ProofSyntax.pretty_proof;
2008-06-18, by wenzelm
removed obsolete term reading operations (cf. old_goals.ML for legacy emulations);
2008-06-18, by wenzelm
added emulations for simple_read_term/read_term/read_prop (formerly in sign.ML);
2008-06-18, by wenzelm
removed obsolete read_def_cterms/read_cterm;
2008-06-18, by wenzelm
load proof term operations later;
2008-06-18, by wenzelm
more antiquotations;
2008-06-18, by wenzelm
OldGoals.read_prop;
2008-06-18, by wenzelm
OldGoals.simple_read_term;
2008-06-18, by wenzelm
simplified Abel_Cancel setup;
2008-06-18, by wenzelm
updated generated file;
2008-06-18, by wenzelm
pervasive cut_inst_tac;
2008-06-18, by wenzelm
added a progress lemma and tuned some comments
2008-06-17, by urbanc
* Rules and tactics that read instantiations now demand a proper context;
2008-06-16, by wenzelm
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
2008-06-16, by wenzelm
renamed rename_params_tac to rename_tac;
2008-06-16, by wenzelm
removed obsolete global instantiation tactics (cf. Isar/rule_insts.ML);
2008-06-16, by wenzelm
removed obsolete no_qed, quick_and_dirty_prove_goalw_cterm;
2008-06-16, by wenzelm
removed obsolete global read_insts/read_instantiate (cf. Isar/rule_insts.ML);
2008-06-16, by wenzelm
inst1_tac: proper context;
2008-06-16, by wenzelm
pervasive RuleInsts;
2008-06-16, by wenzelm
updated generated file;
2008-06-16, by wenzelm
converted ML proofs;
2008-06-16, by wenzelm
added read_instantiate;
2008-06-16, by wenzelm
ML tactic: do not abstract over context again;
2008-06-16, by wenzelm
export eof;
2008-06-16, by wenzelm
removed obsolete inst;
2008-06-16, by wenzelm
atomize: proper context;
2008-06-16, by wenzelm
atomize: proper context;
2008-06-16, by wenzelm
RuleInsts.read_instantiate;
2008-06-16, by wenzelm
ptac/prolog_tac: proper context;
2008-06-16, by wenzelm
allE_Nil: only one copy, proven in regular theory source;
2008-06-16, by wenzelm
deriv_tac/DERIV_tac: proper context;
2008-06-16, by wenzelm
sum3_instantiate: proper context;
2008-06-16, by wenzelm
eliminated OldGoals.inst;
2008-06-16, by wenzelm
updated generated file;
2008-06-16, by wenzelm
method "tactic": only "facts" as bound value;
2008-06-16, by wenzelm
Export a wrapper for all semiring_normalizers
2008-06-16, by chaieb
proper context for tactics derived from res_inst_tac;
2008-06-14, by wenzelm
added ~: and ~=;
2008-06-14, by wenzelm
export subgoal_tac, subgoals_tac, thin_tac;
2008-06-14, by wenzelm
prove: full Variable.declare_term, including constraints;
2008-06-14, by wenzelm
prove_standard: more precises argument passing;
2008-06-14, by wenzelm
InductTacs.case_tac: removed obsolete declare, which is now part of Goal.prove;
2008-06-14, by wenzelm
simplified InductTacs.case_tac/induct_tac;
2008-06-14, by wenzelm
tuned proof;
2008-06-14, by wenzelm
removed obsolete nat_induct_tac -- cannot work without;
2008-06-14, by wenzelm
removed obsolete case_split_tac -- cannot work without;
2008-06-14, by wenzelm
removed unused excluded_middle_tac;
2008-06-14, by wenzelm
updated geenrated file;
2008-06-14, by wenzelm
qualified old res_inst_tac variants;
2008-06-14, by wenzelm
proper context for tactics derived from res_inst_tac;
2008-06-14, by wenzelm
updated generated file;
2008-06-14, by wenzelm
obsolete;
2008-06-14, by wenzelm
certify_term: reject qualified frees;
2008-06-14, by wenzelm
removed experimental Poplog/PML support;
2008-06-14, by wenzelm
removed obsolete ML_SUFFIX;
2008-06-14, by wenzelm
removed experimental Poplog/PML support;
2008-06-14, by wenzelm
removed obsolete ML_SUFFIX;
2008-06-14, by wenzelm
removed exotic 'token_translation' command;
2008-06-14, by wenzelm
proper name for LinearQuantifierElim;
2008-06-14, by wenzelm
removed old theorem database;
2008-06-14, by wenzelm
map_const: soft version, no failure here (recovers hiding of consts, because a hidden name is illegal and rejected later);
2008-06-13, by wenzelm
hide: delete all accesses from extra names -- reduces ambiguity in extern;
2008-06-13, by wenzelm
map_const: soft version, no failure here;
2008-06-13, by wenzelm
skolem_fact/thm: uniform numbering, even for singleton list;
2008-06-13, by wenzelm
hide (open);
2008-06-13, by wenzelm
no_notation instead of hide;
2008-06-13, by wenzelm
* Recovered hiding of consts;
2008-06-13, by wenzelm
updated generated file;
2008-06-13, by wenzelm
back to CodeTarget.code_width;
2008-06-13, by wenzelm
hide -> hide (open)
2008-06-13, by nipkow
use regular error function;
2008-06-12, by wenzelm
add lemma finite_image_approx; remove unnecessary sort annotations
2008-06-12, by huffman
change orientation of fix_eqI and convert to rule_format;
2008-06-12, by huffman
export just one setup function;
2008-06-12, by wenzelm
removed obsolete skolem declarations -- done by Theory.at_end;
2008-06-12, by wenzelm
tuned setup;
2008-06-12, by wenzelm
remove unnecessary import of Ffun;
2008-06-12, by huffman
imports Ffun
2008-06-12, by huffman
ResAxioms.cnf_axiom/cnf_rules_pairs: pass explicit theory context;
2008-06-12, by wenzelm
ResAxioms.cnf_axiom/cnf_rules_pairs: pass explicit theory context;
2008-06-12, by wenzelm
sane versions of (qualified_)thms_of_thy;
2008-06-12, by wenzelm
Facts.dest/export_static: content difference;
2008-06-12, by wenzelm
dest/export_static: content difference;
2008-06-12, by wenzelm
declare_skofuns/skolem: canonical argument order;
2008-06-12, by wenzelm
Facts.dest/export_static: content difference;
2008-06-12, by wenzelm
correction
2008-06-12, by nipkow
tuned
2008-06-12, by nipkow
Removed hide swap
2008-06-12, by nipkow
fixed type
2008-06-12, by nipkow
lemma modified
2008-06-12, by nipkow
typo
2008-06-12, by nipkow
had to add rule: because induct_tac no longer works correctly
2008-06-12, by nipkow
Hid swap
2008-06-12, by nipkow
some reformatting;
2008-06-12, by wenzelm
added CK_Machine to the nominal section
2008-06-12, by urbanc
soundness and completeness proofs for a CK machine as
2008-06-12, by urbanc
emoved the parts that deal with the CK machine to a new theory
2008-06-12, by urbanc
tuned header and comments
2008-06-12, by urbanc
OldGoals.inst;
2008-06-11, by wenzelm
Drule.read_instantiate;
2008-06-11, by wenzelm
qualified inst;
2008-06-11, by wenzelm
qualified types_sorts, read_insts etc.;
2008-06-11, by wenzelm
Drule.types_sorts;
2008-06-11, by wenzelm
OldGoals.inst;
2008-06-11, by wenzelm
Drule.read_instantiate;
2008-06-11, by wenzelm
changed pred_congs: merely cover pred1_cong pred2_cong pred3_cong;
2008-06-11, by wenzelm
removed obsolete/unused pred_congs;
2008-06-11, by wenzelm
tuned comments;
2008-06-11, by wenzelm
converted ML proofs from simpdata.ML;
2008-06-11, by wenzelm
removed dead code;
2008-06-11, by wenzelm
RuleInsts.res_inst_tac with proper context;
2008-06-11, by wenzelm
more antiquotations;
2008-06-11, by wenzelm
tuned;
2008-06-11, by wenzelm
explicit rule for induct_tac
2008-06-11, by haftmann
tuned spacing;
2008-06-10, by wenzelm
updated generated file;
2008-06-10, by wenzelm
* Attributes cases, induct, coinduct support del option.
2008-06-10, by wenzelm
added del attributes;
2008-06-10, by wenzelm
back to original import order -- thanks to proper deletion of nat cases/induct rules from type_definition;
2008-06-10, by wenzelm
proper deletion of nat cases/induct rules from type_definition;
2008-06-10, by wenzelm
fixed spelling (Where is WordExamples.thy anyway?);
2008-06-10, by wenzelm
recovered nat_induct as default for induct_tac;
2008-06-10, by wenzelm
more robust declaration of nat_induct;
2008-06-10, by wenzelm
reordering of imports ensures that nat_induct stay in front;
2008-06-10, by wenzelm
adhoc fix of induct_tac: rule nat_induct;
2008-06-10, by wenzelm
case_tac: accomodate change in bound variable name;
2008-06-10, by wenzelm
nat_induct_tac (works without context);
2008-06-10, by wenzelm
moved case_tac/induct_tac to induct_tacs.ML -- no longer hardwired into datatype package;
2008-06-10, by wenzelm
added nat_induct_tac (works without context);
2008-06-10, by wenzelm
InductTacs.case_tac with proper context and proper declaration of local variable;
2008-06-10, by wenzelm
added HOL/Tools/induct_tacs.ML;
2008-06-10, by wenzelm
eliminated obsolete case_split_thm -- use case_split;
2008-06-10, by wenzelm
tuned proofs -- case_tac *is* available here;
2008-06-10, by wenzelm
updated generated file;
2008-06-10, by wenzelm
case_tac/induct_tac: use same declarations as cases/induct;
2008-06-10, by wenzelm
proper news header;
2008-06-10, by wenzelm
removed obsolete read_idents;
2008-06-10, by wenzelm
added (e)res_inst_tac;
2008-06-10, by wenzelm
focus: actually declare constraints for local parameters;
2008-06-10, by wenzelm
tuned proofs;
2008-06-10, by wenzelm
case_split_tac (works without context);
2008-06-10, by wenzelm
tuned;
2008-06-10, by wenzelm
eliminated obsolete case_split_thm -- use case_split;
2008-06-10, by wenzelm
Unstructured induction and cases analysis for Isabelle/HOL.
2008-06-10, by wenzelm
dropped instance with attached definitions
2008-06-10, by haftmann
polished interface of datatype package
2008-06-10, by haftmann
adjusted some proofs involving inats
2008-06-10, by haftmann
refactoring; addition, numerals
2008-06-10, by haftmann
more instantiation
2008-06-10, by haftmann
whitespace tuning
2008-06-10, by haftmann
localized Least in Orderings.thy
2008-06-10, by haftmann
removed some dubious code lemmas
2008-06-10, by haftmann
slightly tuning of some proofs involving case distinction and induction on natural numbers and similar
2008-06-10, by haftmann
rep_datatype command now takes list of constructors as input arguments
2008-06-10, by haftmann
major refactorings in code generator modules
2008-06-10, by haftmann
updated
2008-06-10, by haftmann
slightly tuning of some proofs involving case distinction and induction on natural numbers and similar
2008-06-10, by haftmann
DatatypePackage.case_tac;
2008-06-09, by wenzelm
DatatypePackage.distinct_simproc;
2008-06-09, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip