author | wenzelm |
Wed, 30 Mar 2016 19:25:04 +0200 | |
changeset 62764 | ff3b8e4079bd |
parent 60758 | d8d85a8172b5 |
child 69605 | a96320074298 |
permissions | -rw-r--r-- |
55085
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
1 |
(* Title: HOL/Fun_Def_Base.thy |
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
2 |
Author: Alexander Krauss, TU Muenchen |
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
3 |
*) |
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
4 |
|
60758 | 5 |
section \<open>Function Definition Base\<close> |
55085
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
6 |
|
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
7 |
theory Fun_Def_Base |
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
8 |
imports Ctr_Sugar Set Wellfounded |
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
9 |
begin |
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
10 |
|
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
11 |
ML_file "Tools/Function/function_lib.ML" |
57959 | 12 |
named_theorems termination_simp "simplification rules for termination proofs" |
55085
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
13 |
ML_file "Tools/Function/function_common.ML" |
58816 | 14 |
ML_file "Tools/Function/function_context_tree.ML" |
15 |
||
16 |
attribute_setup fundef_cong = |
|
17 |
\<open>Attrib.add_del Function_Context_Tree.cong_add Function_Context_Tree.cong_del\<close> |
|
18 |
"declaration of congruence rule for function definitions" |
|
19 |
||
55968 | 20 |
ML_file "Tools/Function/sum_tree.ML" |
55085
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
21 |
|
0e8e4dc55866
moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
blanchet
parents:
diff
changeset
|
22 |
end |