Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-3000
-1000
-120
+120
+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.
obtain;
2000-07-30, by wenzelm
added split_bind_asm, bind_splits;
2000-07-30, by wenzelm
adapted obtain;
2000-07-30, by wenzelm
removed equalityCE;
2000-07-30, by wenzelm
added atomic_Trueprop;
2000-07-30, by wenzelm
updated ObtainFun;
2000-07-30, by wenzelm
'def': no constraint on variable;
2000-07-30, by wenzelm
exporter setup for context elements;
2000-07-30, by wenzelm
export RANGE, hard_asm_tac, soft_asm_tac;
2000-07-30, by wenzelm
turned into plain context element;
2000-07-30, by wenzelm
local_def(_i): no constraint on var;
2000-07-30, by wenzelm
local_def(_i): no constraint on var;
2000-07-30, by wenzelm
def: no constraint on var;
2000-07-30, by wenzelm
added is_judgment;
2000-07-30, by wenzelm
ObtainFun (generalized existence reasoning);
2000-07-30, by wenzelm
ThmDeps.enable;
2000-07-30, by wenzelm
added sign_of_cterm;
2000-07-30, by wenzelm
Logic.goal_const;
2000-07-30, by wenzelm
replaced "Sessions" by "Root";
2000-07-28, by wenzelm
apply. -> by
2000-07-28, by nipkow
* HOL/While
2000-07-28, by nipkow
added theory While;
2000-07-27, by wenzelm
export has_internal;
2000-07-27, by wenzelm
added thm_deps;
2000-07-27, by wenzelm
added enter_forward_proof;
2000-07-27, by wenzelm
export write_graph;
2000-07-27, by wenzelm
begin_theory: store *copy* of initial theory;
2000-07-27, by wenzelm
tuned;
2000-07-27, by wenzelm
intro_elim_tac: bimatch_from;
2000-07-27, by wenzelm
While functional for defining tail-recursive functions
2000-07-26, by nipkow
*** empty log message ***
2000-07-26, by nipkow
tuned msg;
2000-07-25, by wenzelm
Corrected example which still used old primrec syntax.
2000-07-25, by berghofe
Replaced force by fast because force may now take forever to fail
2000-07-25, by nipkow
new constant same_fst
2000-07-25, by nipkow
by (CLASIMPSET auto_tac);
2000-07-25, by wenzelm
added clarify method;
2000-07-25, by wenzelm
added clarsimp method;
2000-07-25, by wenzelm
tuned;
2000-07-25, by wenzelm
removed slow, slow_best methods;
2000-07-25, by wenzelm
* Isar/Provers: intro/elim/dest attributes: changed
2000-07-25, by wenzelm
rearranged setup of arithmetic procedures, avoiding global reference values;
2000-07-25, by wenzelm
lemmas [arith_split] = abs_split (*belongs to theory RealAbs*);
2000-07-25, by wenzelm
do nat pass theory value, but sg_ref;
2000-07-25, by wenzelm
avoid referencing thy value;
2000-07-25, by wenzelm
avoid referencing thy value;
2000-07-25, by wenzelm
tuned deps;
2000-07-25, by wenzelm
tuned;
2000-07-24, by wenzelm
changed deps;
2000-07-24, by wenzelm
rename_numerals: use implicit theory context;
2000-07-24, by wenzelm
avoid referencing thy value;
2000-07-24, by wenzelm
avoid referencing thy value;
2000-07-24, by wenzelm
avoid referencing thy value;
2000-07-24, by wenzelm
simpset_of NatDef.thy (why anyway?);
2000-07-24, by wenzelm
avoid referencing thy value;
2000-07-24, by wenzelm
avoid referencing thy value;
2000-07-24, by wenzelm
tuned comment;
2000-07-24, by wenzelm
avoid global references;
2000-07-24, by wenzelm
do not pass theory values, but sg_ref;
2000-07-24, by wenzelm
Drule.merge_rules;
2000-07-24, by wenzelm
get_names: topologically sorted;
2000-07-23, by wenzelm
removed all_sessions.graph;
2000-07-23, by wenzelm
removed all_sessions;
2000-07-23, by wenzelm
disallow duplicates in session identifiers;
2000-07-23, by wenzelm
assimilated;
2000-07-23, by wenzelm
tuned HeapFun;
2000-07-23, by wenzelm
tuned ThmHeap;
2000-07-23, by wenzelm
removed selector syntax -- improper tuples are broken beyond repair :-(
2000-07-23, by wenzelm
elim?;
2000-07-23, by wenzelm
classical atts now intro! / intro / intro?;
2000-07-23, by wenzelm
renamed "Directories" to "Sessions";
2000-07-23, by wenzelm
tuned;
2000-07-23, by wenzelm
improved error msg;
2000-07-22, by wenzelm
added ex_someI
2000-07-21, by nipkow
much tidying in connection with the 2nd UNITY paper
2000-07-21, by paulson
strengthened force_tac by using new first_best_tac
2000-07-21, by oheimb
removed safe_asm_full_simp_tac
2000-07-21, by oheimb
added map_upd_nonempty, also to simpset
2000-07-21, by oheimb
removed weaker variant of subset_insert_iff
2000-07-21, by oheimb
removed safe_asm_full_simp_tac, added generic_simp_tac
2000-07-21, by oheimb
Updating of some comments
2000-07-21, by prensani
*** empty log message ***
2000-07-21, by nipkow
Univ no longer requires Arith (really it never did)
2000-07-21, by paulson
tuned;
2000-07-20, by wenzelm
corrected header
2000-07-19, by oheimb
changed / to // for quotienting
2000-07-19, by paulson
changed / to // for quotienting; general tidying
2000-07-19, by paulson
renamed // to / (which is what we want anyway) to avoid clash with the new
2000-07-19, by paulson
deleted redundant proof
2000-07-19, by paulson
// change; also moved entry for AddIffs
2000-07-19, by paulson
addsplits [split_if];
2000-07-18, by wenzelm
theorems foo.splits = foo.split foo.split_asm;
2000-07-18, by wenzelm
removed obsolete expand_if = split_if;
2000-07-18, by wenzelm
* HOL: removed obsolete expand_if = split_if; theorems if_splits =
2000-07-18, by wenzelm
* HOL: removed obsolete expand_if = split_if; theorems if_splits =
2000-07-18, by wenzelm
replaced arities by instance;
2000-07-18, by wenzelm
MicroJava structure changed
2000-07-18, by kleing
consts: include *all* names;
2000-07-17, by wenzelm
tuded presentation;
2000-07-17, by bauerg
AddXIs [UnI1, UnI2];
2000-07-17, by wenzelm
flat instruction set, op. semantics now in JVMExecInstr.thy
2000-07-17, by kleing
flat instruction set
2000-07-17, by kleing
10pt
2000-07-17, by bauerg
- xsymbols for
2000-07-17, by bauerg
strip_prod_type = HOLogic.prodT_factors;
2000-07-16, by wenzelm
AST translation rules no longer require constant head on LHS;
2000-07-16, by wenzelm
fixed nested prod syntax;
2000-07-16, by wenzelm
use split_tupled_all;
2000-07-16, by wenzelm
use pair_tac;
2000-07-16, by wenzelm
adapted tuple syntax;
2000-07-16, by wenzelm
tuned;
2000-07-16, by wenzelm
use pair_tac;
2000-07-16, by wenzelm
use split syntax;
2000-07-16, by wenzelm
fixed tuple translations;
2000-07-16, by wenzelm
defs (overloaded);
2000-07-16, by wenzelm
added is_unitT;
2000-07-16, by wenzelm
instance unit :: finite;
2000-07-16, by wenzelm
more robust tuple syntax (still improper, though!);
2000-07-16, by wenzelm
improved unit theory: unit_all_eq1, unit_all_eq2, split_all_tac;
2000-07-16, by wenzelm
added syntax for proper / improper selector functions;
2000-07-16, by wenzelm
less
more
|
(0)
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip