hoelzl [Wed, 23 Sep 2009 13:31:38 +0200] rev 32651
Undo errornous commit of Statespace change
hoelzl [Wed, 23 Sep 2009 13:17:17 +0200] rev 32650
correct variable order in approximate-method
paulson [Wed, 23 Sep 2009 11:06:32 +0100] rev 32649
merged
paulson [Wed, 23 Sep 2009 11:05:28 +0100] rev 32648
Correct chasing of type variable instantiations during type unification.
The following theory should not raise exception TERM:
constdefs
somepredicate :: "(('b => 'b) => ('a => 'a))
=> 'a => 'b => bool"
"somepredicate upd v x == True"
lemma somepredicate_idI:
"somepredicate id (f v) v"
by (simp add: somepredicate_def)
lemma somepredicate_triv:
"somepredicate upd v x ==> somepredicate upd v x"
by assumption
lemmas somepredicate_triv [OF somepredicate_idI]
lemmas st' = somepredicate_triv[where v="h :: nat => bool"]
lemmas st2 = st'[OF somepredicate_idI]
haftmann [Wed, 23 Sep 2009 11:33:52 +0200] rev 32647
hide newly introduced constants
Philipp Meyer [Tue, 22 Sep 2009 11:26:46 +0200] rev 32646
used standard fold function and type aliases
Philipp Meyer [Mon, 21 Sep 2009 15:05:26 +0200] rev 32645
sos method generates and uses proof certificates
wenzelm [Tue, 22 Sep 2009 20:25:31 +0200] rev 32644
full reserve of worker threads -- for improved CPU utilization;
haftmann [Tue, 22 Sep 2009 15:38:12 +0200] rev 32643
merged
haftmann [Tue, 22 Sep 2009 15:36:55 +0200] rev 32642
be more cautious wrt. simp rules: inf_absorb1, inf_absorb2, sup_absorb1, sup_absorb2 are no simp rules by default any longer
krauss [Tue, 22 Sep 2009 15:12:45 +0200] rev 32641
tail -n 20: more helpful output if make fails
haftmann [Tue, 22 Sep 2009 08:58:08 +0200] rev 32640
corrected order of type variables in code equations; more precise certificate for cases
Christian Urban <urbanc@in.tum.de> [Mon, 21 Sep 2009 16:16:16 +0200] rev 32639
merged
Christian Urban <urbanc@in.tum.de> [Mon, 21 Sep 2009 15:02:23 +0200] rev 32638
tuned some proofs
haftmann [Mon, 21 Sep 2009 16:11:36 +0200] rev 32637
merged
haftmann [Mon, 21 Sep 2009 16:01:38 +0200] rev 32636
added session theory for Bali and Nominal_Examples
haftmann [Mon, 21 Sep 2009 16:01:30 +0200] rev 32635
added session theory for Nominal_Examples
haftmann [Mon, 21 Sep 2009 16:00:53 +0200] rev 32634
added session theory for Bali
haftmann [Mon, 21 Sep 2009 16:00:34 +0200] rev 32633
adjusted to new Number Theory scenario
haftmann [Mon, 21 Sep 2009 15:33:40 +0200] rev 32632
added session entry point theories
haftmann [Mon, 21 Sep 2009 15:33:40 +0200] rev 32631
common base for protocols with symmetric keys
haftmann [Mon, 21 Sep 2009 15:33:39 +0200] rev 32630
tuned header
haftmann [Mon, 21 Sep 2009 14:22:32 +0200] rev 32629
isarified proof
wenzelm [Mon, 21 Sep 2009 16:07:20 +0200] rev 32628
fixed permissions -- this is a script, not an executable;
wenzelm [Mon, 21 Sep 2009 16:06:52 +0200] rev 32627
tuned;
boehmes [Mon, 21 Sep 2009 13:42:36 +0200] rev 32626
deleted unused file
haftmann [Mon, 21 Sep 2009 12:23:05 +0200] rev 32625
merged
haftmann [Mon, 21 Sep 2009 12:22:53 +0200] rev 32624
entry point theory for examples; reactivated half-dead example
boehmes [Mon, 21 Sep 2009 11:15:55 +0200] rev 32623
merged
boehmes [Mon, 21 Sep 2009 11:15:21 +0200] rev 32622
corrected remote SMT solver invocation
haftmann [Mon, 21 Sep 2009 10:58:25 +0200] rev 32621
theory entry point for session Hoare_Parallel (now also with proper underscore)
boehmes [Mon, 21 Sep 2009 08:45:31 +0200] rev 32620
merged
boehmes [Mon, 21 Sep 2009 08:34:56 +0200] rev 32619
tuned author
boehmes [Fri, 18 Sep 2009 18:13:19 +0200] rev 32618
added new method "smt": an oracle-based connection to external SMT solvers
wenzelm [Sun, 20 Sep 2009 19:17:33 +0200] rev 32617
tuned tracing;
wenzelm [Sun, 20 Sep 2009 18:37:55 +0200] rev 32616
scheduler backdoor: 9999 means 1 worker;
wenzelm [Sun, 20 Sep 2009 18:15:07 +0200] rev 32615
Hilbert_Classical: more precise control of parallel_proofs;
wenzelm [Sun, 20 Sep 2009 17:23:23 +0200] rev 32614
actually observe Multithreading.enabled (cf. d302f1c9e356);
nipkow [Sat, 19 Sep 2009 10:19:34 +0200] rev 32613
merged
nipkow [Sat, 19 Sep 2009 10:19:12 +0200] rev 32612
restructured code
haftmann [Sat, 19 Sep 2009 07:35:27 +0200] rev 32611
merged
haftmann [Fri, 18 Sep 2009 16:00:56 +0200] rev 32610
rewrite premises in tactical proof also with inf_fun_eq and inf_bool_eq: attempt to allow user to use inf [=>] and inf [bool] in his specs
nipkow [Fri, 18 Sep 2009 23:08:53 +0200] rev 32609
modified minimization log
nipkow [Fri, 18 Sep 2009 14:40:24 +0200] rev 32608
merged
nipkow [Fri, 18 Sep 2009 14:40:06 +0200] rev 32607
skip &&& goals
haftmann [Fri, 18 Sep 2009 14:09:38 +0200] rev 32606
INTER and UNION are mere abbreviations for INFI and SUPR
haftmann [Fri, 18 Sep 2009 09:35:23 +0200] rev 32605
simplified proof
haftmann [Fri, 18 Sep 2009 09:07:51 +0200] rev 32604
partially isarified proof
haftmann [Fri, 18 Sep 2009 09:07:50 +0200] rev 32603
tuned const_name antiquotations
haftmann [Fri, 18 Sep 2009 09:07:49 +0200] rev 32602
more antiquotations
haftmann [Fri, 18 Sep 2009 09:07:48 +0200] rev 32601
be more cautious wrt. simp rules: sup1_iff, sup2_iff, inf1_iff, inf2_iff, SUP1_iff, SUP2_iff, INF1_iff, INF2_iff are no longer simp by default
haftmann [Fri, 18 Sep 2009 07:54:26 +0200] rev 32600
tuned NEWS, added CONTRIBUTORS
nipkow [Thu, 17 Sep 2009 19:13:22 +0200] rev 32599
merged
nipkow [Thu, 17 Sep 2009 19:13:07 +0200] rev 32598
removed misleading log line
paulson [Thu, 17 Sep 2009 15:04:46 +0100] rev 32597
NEWS: New method metisFT
paulson [Thu, 17 Sep 2009 14:59:58 +0100] rev 32596
New theorems for proving equalities and inclusions involving unions